Groups lectures (#25)

This commit is contained in:
Patrick Stevens
2019-02-19 08:24:38 +00:00
committed by GitHub
parent d2192c72d9
commit 674aae49cd
8 changed files with 593 additions and 71 deletions

10
DecidableSet.agda Normal file
View 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))