Skip to content

Commit

Permalink
feat(group_theory/nilpotent): add nilpotent implies normalizer condit…
Browse files Browse the repository at this point in the history
…ion (#11586)
  • Loading branch information
nomeata committed Feb 10, 2022
1 parent c3f6fce commit 1373d54
Show file tree
Hide file tree
Showing 2 changed files with 27 additions and 0 deletions.
23 changes: 23 additions & 0 deletions src/group_theory/nilpotent.lean
Expand Up @@ -726,3 +726,26 @@ begin
end

end classical

lemma normalizer_condition_of_is_nilpotent [h : is_nilpotent G] : normalizer_condition G :=
begin
-- roughly based on https://groupprops.subwiki.org/wiki/Nilpotent_implies_normalizer_condition
rw normalizer_condition_iff_only_full_group_self_normalizing,
unfreezingI
{ induction h using nilpotent_center_quotient_ind with G' _ _ G' _ _ ih;
clear _inst_1 G; rename G' → G, },
{ rintros H -, apply subsingleton.elim, },
{ intros H hH,

have hch : center G ≤ H := subgroup.center_le_normalizer.trans (le_of_eq hH),
have hkh : (mk' (center G)).ker ≤ H, by simpa using hch,
have hsur : function.surjective (mk' (center G)), by exact surjective_quot_mk _,

let H' := H.map (mk' (center G)),
have hH' : H'.normalizer = H',
{ apply comap_injective hsur,
rw [comap_normalizer_eq_of_surjective _ hsur, comap_map_eq_self hkh],
exact hH, },
apply map_injective_of_ker_le (mk' (center G)) hkh le_top,
exact (ih H' hH').trans (symm (map_top_of_surjective _ hsur)), },
end
4 changes: 4 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -981,6 +981,10 @@ end
@[simp, to_additive] lemma map_bot (f : G →* N) : (⊥ : subgroup G).map f = ⊥ :=
(gc_map_comap f).l_bot

@[simp, to_additive] lemma map_top_of_surjective (f : G →* N) (h : function.surjective f) :
subgroup.map f ⊤ = ⊤ :=
by {rw eq_top_iff, intros x hx, obtain ⟨y, hy⟩ := (h x), exact ⟨y, trivial, hy⟩ }

@[simp, to_additive] lemma comap_top (f : G →* N) : (⊤ : subgroup N).comap f = ⊤ :=
(gc_map_comap f).u_top

Expand Down

0 comments on commit 1373d54

Please sign in to comment.