Finite permutations (#23)

This commit is contained in:
Patrick Stevens
2019-02-18 08:30:26 +00:00
committed by GitHub
parent c35fa90951
commit 0650021db1
12 changed files with 454 additions and 109 deletions

View File

@@ -67,6 +67,8 @@ module Setoids.Setoids where
field
inj : SetoidInjection S T f
surj : SetoidSurjection S T f
wellDefined : {x y : A} Setoid.__ S x y Setoid.__ T (f x) (f y)
wellDefined = SetoidInjection.wellDefined inj
record SetoidsBiject {a b c d : _} {A : Set a} {B : Set b} (S : Setoid {a} {c} A) (T : Setoid {b} {d} B) : Set (a b c d) where
field