Skip to content

Commit

Permalink
feat(group_theory/coset): rw lemmas involving quotient_group.mk (#8957)
Browse files Browse the repository at this point in the history
When doing computations with quotient groups, I found these lemmas to be helpful when rewriting.
  • Loading branch information
tb65536 committed Sep 2, 2021
1 parent baefdf3 commit 55a7d38
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/group_theory/coset.lean
Expand Up @@ -295,6 +295,14 @@ instance (s : subgroup α) : inhabited (quotient s) :=
protected lemma eq {a b : α} : (a : quotient s) = b ↔ a⁻¹ * b ∈ s :=
quotient.eq'

@[to_additive quotient_add_group.eq']
lemma eq' {a b : α} : (mk a : quotient s) = mk b ↔ a⁻¹ * b ∈ s :=
quotient_group.eq

@[to_additive quotient_add_group.out_eq']
lemma out_eq' (a : quotient s) : mk a.out' = a :=
quotient.out_eq' a

@[to_additive]
lemma eq_class_eq_left_coset (s : subgroup α) (g : α) :
{x : α | (x : quotient s) = g} = left_coset g s :=
Expand Down

0 comments on commit 55a7d38

Please sign in to comment.