Skip to content

Commit 1f3a116

Browse files
committed
feat(GroupTheory/Complement): Quotient of complementary subgroup (#20101)
If `H` and `K` are complementary with `K` normal, then `G/K` is isomorphic to `H`.
1 parent 1f090b0 commit 1f3a116

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

Mathlib/GroupTheory/Complement.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -613,6 +613,14 @@ theorem IsComplement'.disjoint (h : IsComplement' H K) : Disjoint H K :=
613613
theorem IsComplement'.index_eq_card (h : IsComplement' H K) : K.index = Nat.card H :=
614614
(card_left_transversal h).symm
615615

616+
/-- If `H` and `K` are complementary with `K` normal, then `G ⧸ K` is isomorphic to `H`. -/
617+
@[simps!]
618+
noncomputable def IsComplement'.QuotientMulEquiv [K.Normal] (h : H.IsComplement' K) :
619+
G ⧸ K ≃* H :=
620+
MulEquiv.symm
621+
{ (MemLeftTransversals.toEquiv h).symm with
622+
map_mul' := fun _ _ ↦ rfl }
623+
616624
theorem IsComplement.card_mul (h : IsComplement S T) :
617625
Nat.card S * Nat.card T = Nat.card G :=
618626
(Nat.card_prod _ _).symm.trans (Nat.card_eq_of_bijective _ h)

0 commit comments

Comments
 (0)