Skip to content

Commit

Permalink
chore(group_theory/quotient_group): Tag lemmas with @[to_additive] (#…
Browse files Browse the repository at this point in the history
…9771)

Adds `@[to_additive]` to a couple lemmas.
  • Loading branch information
tb65536 committed Oct 17, 2021
1 parent a1a05ad commit 7aa431c
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/group_theory/quotient_group.lean
Expand Up @@ -414,11 +414,12 @@ end third_iso_thm

section trivial

lemma subsingleton_quotient_top : subsingleton (quotient_group.quotient (⊤ : subgroup G)) :=
@[to_additive] lemma subsingleton_quotient_top :
subsingleton (quotient_group.quotient (⊤ : subgroup G)) :=
trunc.subsingleton

/-- If the quotient by a subgroup gives a singleton then the subgroup is the whole group. -/
lemma subgroup_eq_top_of_subsingleton (H : subgroup G)
@[to_additive] lemma subgroup_eq_top_of_subsingleton (H : subgroup G)
(h : subsingleton (quotient_group.quotient H)) : H = ⊤ :=
top_unique $ λ x _,
have this : 1⁻¹ * x ∈ H := quotient_group.eq.1 (subsingleton.elim _ _),
Expand Down

0 comments on commit 7aa431c

Please sign in to comment.