Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): Bottom subgroup has unique element (
Browse files Browse the repository at this point in the history
…#9734)

Adds instance for `unique (⊥ : subgroup G)`.
  • Loading branch information
tb65536 committed Oct 16, 2021
1 parent 1766588 commit 150bbea
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -408,6 +408,8 @@ instance : inhabited (subgroup G) := ⟨⊥⟩

@[simp, to_additive] lemma coe_bot : ((⊥ : subgroup G) : set G) = {1} := rfl

@[to_additive] instance : unique (⊥ : subgroup G) := ⟨⟨1⟩, λ g, subtype.ext g.2

@[to_additive] lemma eq_bot_iff_forall : H = ⊥ ↔ ∀ x ∈ H, x = (1 : G) :=
begin
rw set_like.ext'_iff,
Expand Down

0 comments on commit 150bbea

Please sign in to comment.