File tree Expand file tree Collapse file tree 1 file changed +8
-0
lines changed
Expand file tree Collapse file tree 1 file changed +8
-0
lines changed Original file line number Diff line number Diff line change @@ -613,6 +613,14 @@ theorem IsComplement'.disjoint (h : IsComplement' H K) : Disjoint H K :=
613613theorem 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+
616624theorem 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)
You can’t perform that action at this time.
0 commit comments