Skip to content

Commit

Permalink
feat(group_theory/nilpotent): add upper_central_series_eq_top_iff_nil…
Browse files Browse the repository at this point in the history
…potency_class_le (#11670)

and the analogue for the lower central series.
  • Loading branch information
nomeata committed Jan 28, 2022
1 parent 7a485b1 commit 92c64c4
Showing 1 changed file with 25 additions and 0 deletions.
25 changes: 25 additions & 0 deletions src/group_theory/nilpotent.lean
Expand Up @@ -354,6 +354,18 @@ lemma upper_central_series_nilpotency_class :
upper_central_series G (group.nilpotency_class G) = ⊤ :=
nat.find_spec (is_nilpotent.nilpotent G)

lemma upper_central_series_eq_top_iff_nilpotency_class_le {n : ℕ} :
(upper_central_series G n = ⊤) ↔ (group.nilpotency_class G ≤ n) :=
begin
split,
{ intro h,
exact (nat.find_le h), },
{ intro h,
apply eq_top_iff.mpr,
rw ← upper_central_series_nilpotency_class,
exact (upper_central_series_mono _ h), }
end

/-- The nilpotency class of a nilpotent `G` is equal to the smallest `n` for which an ascending
central series reaches `G` in its `n`'th term. -/
lemma least_ascending_central_series_length_eq_nilpotency_class :
Expand Down Expand Up @@ -405,6 +417,19 @@ begin
exact (nat.find_spec (nilpotent_iff_lower_central_series.mp _))
end

lemma lower_central_series_eq_bot_iff_nilpotency_class_le {n : ℕ} :
(lower_central_series G n = ⊥) ↔ (group.nilpotency_class G ≤ n) :=
begin
split,
{ intro h,
rw ← lower_central_series_length_eq_nilpotency_class,
exact (nat.find_le h), },
{ intro h,
apply eq_bot_iff.mpr,
rw ← lower_central_series_nilpotency_class,
exact (lower_central_series_antitone h), }
end

end classical

lemma lower_central_series_map_subtype_le (H : subgroup G) (n : ℕ) :
Expand Down

0 comments on commit 92c64c4

Please sign in to comment.