Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): Range of inclusion (#9732)
Browse files Browse the repository at this point in the history
If `H ≤ K`, then the range of `inclusion : H → K` is `H` (viewed as a subgroup of `K`).
  • Loading branch information
tb65536 committed Oct 16, 2021
1 parent 155f8e6 commit aa0d0d4
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -1415,6 +1415,10 @@ range_top_iff_surjective.2 hf
@[simp, to_additive] lemma _root_.subgroup.subtype_range (H : subgroup G) : H.subtype.range = H :=
by { rw [range_eq_map, ← set_like.coe_set_eq, coe_map, subgroup.coe_subtype], ext, simp }

@[simp, to_additive] lemma _root_.subgroup.inclusion_range {H K : subgroup G} (h_le : H ≤ K) :
(inclusion h_le).range = H.subgroup_of K :=
subgroup.ext (λ g, set.ext_iff.mp (set.range_inclusion h_le) g)

/-- Restriction of a group hom to a subgroup of the domain. -/
@[to_additive "Restriction of an `add_group` hom to an `add_subgroup` of the domain."]
def restrict (f : G →* N) (H : subgroup G) : H →* N :=
Expand Down

0 comments on commit aa0d0d4

Please sign in to comment.