Skip to content

Commit

Permalink
feat(group_theory/subgroup) top is a normal subgroup (#4982)
Browse files Browse the repository at this point in the history
  • Loading branch information
alexjbest committed Nov 12, 2020
1 parent 509a224 commit 3f575d7
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/group_theory/subgroup.lean
Expand Up @@ -747,6 +747,9 @@ end normal
@[priority 100, to_additive]
instance bot_normal : normal (⊥ : subgroup G) := ⟨by simp⟩

@[priority 100, to_additive]
instance top_normal : normal (⊤ : subgroup G) := ⟨λ _ _, mem_top⟩

variable (G)
/-- The center of a group `G` is the set of elements that commute with everything in `G` -/
@[to_additive "The center of a group `G` is the set of elements that commute with everything in `G`"]
Expand Down

0 comments on commit 3f575d7

Please sign in to comment.