mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-22 11:38:38 +00:00
Groups lectures (#25)
This commit is contained in:
10
DecidableSet.agda
Normal file
10
DecidableSet.agda
Normal file
@@ -0,0 +1,10 @@
|
||||
{-# OPTIONS --safe --warning=error #-}
|
||||
|
||||
open import LogicalFormulae
|
||||
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
|
||||
|
||||
module DecidableSet where
|
||||
|
||||
record DecidableSet {a : _} (A : Set a) : Set a where
|
||||
field
|
||||
eq : (a b : A) → ((a ≡ b) || ((a ≡ b) → False))
|
Reference in New Issue
Block a user