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

View File

@@ -58,14 +58,6 @@ module Groups.Groups where
m : y z · e
m = transitive l (wellDefined ~refl invRight)
identityIsUnique : {a b : _} {A : Set a} {S : Setoid {a} {b} A} {_·_ : A A A} (G : Group S _·_) (e : A) ((b : A) (Setoid.__ S (b · e) b)) (Setoid.__ S e (Group.identity G))
identityIsUnique {S = S} {_·_} g thing fb = transitive (symmetric multIdentLeft) (fb e)
where
open Group g renaming (inverse to _^-1) renaming (identity to e)
open Setoid S
open Transitive (Equivalence.transitiveEq eq)
open Symmetric (Equivalence.symmetricEq eq)
replaceGroupOp : {l m : _} {A : Set l} {S : Setoid {l} {m} A} {_·_ : A A A} (G : Group S _·_) {a b c d w x y z : A} (Setoid.__ S a c) (Setoid.__ S b d) (Setoid.__ S w y) (Setoid.__ S x z) Setoid.__ S (a · b) (w · x) Setoid.__ S (c · d) (y · z)
replaceGroupOp {S = S} {_·_} G a~c b~d w~y x~z pr = transitive (symmetric (wellDefined a~c b~d)) (transitive pr (wellDefined w~y x~z))
where