Skip to content

Commit

Permalink
feat(group_theory): generalize normal_map (#17808)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Dec 4, 2022
1 parent 6c5959a commit cc3c8aa
Show file tree
Hide file tree
Showing 2 changed files with 11 additions and 7 deletions.
9 changes: 2 additions & 7 deletions src/group_theory/quotient_group.lean
Expand Up @@ -489,13 +489,8 @@ variables (M : subgroup G) [nM : M.normal]

include nM nN

@[to_additive quotient_add_group.map_normal]
instance map_normal : (M.map (quotient_group.mk' N)).normal :=
{ conj_mem := begin
rintro _ ⟨x, hx, rfl⟩ y,
refine induction_on' y (λ y, ⟨y * x * y⁻¹, subgroup.normal.conj_mem nM x hx y, _⟩),
simp only [mk'_apply, coe_mul, coe_inv]
end }
@[to_additive] instance map_normal : (M.map (quotient_group.mk' N)).normal :=
nM.map _ mk_surjective

variables (h : N ≤ M)

Expand Down
9 changes: 9 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -2230,6 +2230,15 @@ namespace subgroup

variables {N : Type*} [group N] (H : subgroup G)

@[to_additive]
lemma normal.map {H : subgroup G} (h : H.normal) (f : G →* N) (hf : function.surjective f) :
(H.map f).normal :=
begin
rw [← normalizer_eq_top, ← top_le_iff, ← f.range_top_of_surjective hf, f.range_eq_map,
← normalizer_eq_top.2 h],
exact le_normalizer_map _
end

@[to_additive] lemma map_eq_bot_iff {f : G →* N} : H.map f = ⊥ ↔ H ≤ f.ker :=
(gc_map_comap f).l_eq_bot

Expand Down

0 comments on commit cc3c8aa

Please sign in to comment.