Move equiv rels (#46)

This commit is contained in:
Patrick Stevens
2019-09-28 22:24:41 +01:00
committed by GitHub
parent b92e6b2dd8
commit 00ce1dfdf8
20 changed files with 455 additions and 769 deletions

View File

@@ -99,21 +99,3 @@ module Functions where
codom : {a b : _} {A : Set a} {B : Set b} (f : A B) Set b
codom {B = B} f = B
record Reflexive {a b : _} {A : Set a} (r : Rel {a} {b} A) : Set (a lsuc b) where
field
reflexive : {b : A} r b b
record Symmetric {a b : _} {A : Set a} (r : Rel {a} {b} A) : Set (a lsuc b) where
field
symmetric : {b c : A} r b c r c b
record Transitive {a b : _} {A : Set a} (r : Rel {a} {b} A) : Set (a lsuc b) where
field
transitive : {b c d : A} r b c r c d r b d
record Equivalence {a b : _} {A : Set a} (r : Rel {a} {b} A) : Set (a lsuc b) where
field
reflexiveEq : Reflexive r
symmetricEq : Symmetric r
transitiveEq : Transitive r