Skip to content

Commit

Permalink
feat(group_theory/sylow): Sylow subgroups are Hall subgroups (#14624)
Browse files Browse the repository at this point in the history
This PR adds a lemma stating that Sylow subgroups are Hall subgroups (cardinality is coprime to index).
  • Loading branch information
tb65536 committed Jun 11, 2022
1 parent 18936e5 commit 050404a
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/group_theory/sylow.lean
Expand Up @@ -520,6 +520,12 @@ begin
rwa pow_one at key,
end

/-- Sylow subgroups are Hall subgroups. -/
lemma card_coprime_index [fintype G] {p : ℕ} [hp : fact p.prime] (P : sylow p G) :
(card P).coprime (index (P : subgroup G)) :=
let ⟨n, hn⟩ := is_p_group.iff_card.mp P.2 in
hn.symm ▸ (hp.1.coprime_pow_of_not_dvd (not_dvd_index_sylow P index_ne_zero_of_fintype)).symm

lemma ne_bot_of_dvd_card [fintype G] {p : ℕ} [hp : fact p.prime] (P : sylow p G)
(hdvd : p ∣ card G) : (P : subgroup G) ≠ ⊥ :=
begin
Expand Down

0 comments on commit 050404a

Please sign in to comment.