Skip to content

Commit

Permalink
feat(GroupTheory/Complement): Quotient of complementary subgroup (#20101
Browse files Browse the repository at this point in the history
)

If `H` and `K` are complementary with `K` normal, then `G/K` is isomorphic to `H`.
  • Loading branch information
tb65536 committed Dec 20, 2024
1 parent 1f090b0 commit 1f3a116
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Mathlib/GroupTheory/Complement.lean
Original file line number Diff line number Diff line change
Expand Up @@ -613,6 +613,14 @@ theorem IsComplement'.disjoint (h : IsComplement' H K) : Disjoint H K :=
theorem IsComplement'.index_eq_card (h : IsComplement' H K) : K.index = Nat.card H :=
(card_left_transversal h).symm

/-- If `H` and `K` are complementary with `K` normal, then `G ⧸ K` is isomorphic to `H`. -/
@[simps!]
noncomputable def IsComplement'.QuotientMulEquiv [K.Normal] (h : H.IsComplement' K) :
G ⧸ K ≃* H :=
MulEquiv.symm
{ (MemLeftTransversals.toEquiv h).symm with
map_mul' := fun _ _ ↦ rfl }

theorem IsComplement.card_mul (h : IsComplement S T) :
Nat.card S * Nat.card T = Nat.card G :=
(Nat.card_prod _ _).symm.trans (Nat.card_eq_of_bijective _ h)
Expand Down

0 comments on commit 1f3a116

Please sign in to comment.