Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 591ff3a

Browse files
committed
feat(group_theory/subgroup): Subgroup of subgroup is isomorphic to itself (#9204)
If `H ≤ K`, then `H` as a subgroup of `K` is isomorphic to `H`.
1 parent 463089d commit 591ff3a

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

src/group_theory/subgroup.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -896,6 +896,16 @@ ext $ λ x, and_iff_right_of_imp (λ _, x.prop)
896896
lemma comap_subtype_inf_right {H K : subgroup G} : comap K.subtype (H ⊓ K) = comap K.subtype H :=
897897
ext $ λ x, and_iff_left_of_imp (λ _, x.prop)
898898

899+
/-- If `H ≤ K`, then `H` as a subgroup of `K` is isomorphic to `H`. -/
900+
@[to_additive "If `H ≤ K`, then `H` as a subgroup of `K` is isomorphic to `H`.", simps]
901+
def comap_subtype_equiv_of_le {G : Type*} [group G] {H K : subgroup G} (h : H ≤ K) :
902+
H.comap K.subtype ≃* H :=
903+
{ to_fun := λ g, ⟨g.1, g.2⟩,
904+
inv_fun := λ g, ⟨⟨g.1, h g.2⟩, g.2⟩,
905+
left_inv := λ g, subtype.ext (subtype.ext rfl),
906+
right_inv := λ g, subtype.ext rfl,
907+
map_mul' := λ g h, rfl }
908+
899909
/-- For any subgroups `H` and `K`, view `H ⊓ K` as a subgroup of `K`. -/
900910
@[to_additive "For any subgroups `H` and `K`, view `H ⊓ K` as a subgroup of `K`."]
901911
def subgroup_of (H K : subgroup G) : subgroup K := H.comap K.subtype

0 commit comments

Comments
 (0)