Skip to content

Commit

Permalink
feat(group_theory/p_group): Bottom subgroup is a p-group (#9190)
Browse files Browse the repository at this point in the history
The bottom subgroup is a p-group.

Name is consistent with `is_p_group.of_card`
  • Loading branch information
tb65536 committed Sep 14, 2021
1 parent 8dffafd commit d3b345d
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/group_theory/p_group.lean
Expand Up @@ -36,6 +36,9 @@ forall_congr (λ g, ⟨λ ⟨k, hk⟩, exists_imp_exists (by exact λ j, Exists.
lemma of_card [fintype G] {n : ℕ} (hG : fintype.card G = p ^ n) : is_p_group p G :=
λ g, ⟨n, by rw [←hG, pow_card_eq_one]⟩

lemma of_bot : is_p_group p (⊥ : subgroup G) :=
of_card (subgroup.card_bot.trans (pow_zero p).symm)

lemma iff_card [fact p.prime] [fintype G] :
is_p_group p G ↔ ∃ n : ℕ, fintype.card G = p ^ n :=
begin
Expand Down

0 comments on commit d3b345d

Please sign in to comment.