Skip to content

Commit

Permalink
feat(NumberTheory/LSeries/Convergence): add lemma on real-valued seri…
Browse files Browse the repository at this point in the history
…es (#19334)

This is part of the series of PRs leading to Dirichlet's Theorem on primes in AP.

See [here](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/Prerequisites.20for.20PNT.20and.20Dirichlet's.20Thm/near/483303184) on Zulip.
  • Loading branch information
MichaelStollBayreuth committed Nov 21, 2024
1 parent 29b03c8 commit d59b190
Showing 1 changed file with 18 additions and 0 deletions.
18 changes: 18 additions & 0 deletions Mathlib/NumberTheory/LSeries/Convergence.lean
Original file line number Diff line number Diff line change
Expand Up @@ -119,3 +119,21 @@ lemma LSeries.abscissaOfAbsConv_le_one_of_isBigO_one {f : ℕ → ℂ} (h : f =O
convert abscissaOfAbsConv_le_of_isBigO_rpow (x := 0) ?_
· simp only [EReal.coe_zero, zero_add]
· simpa only [Real.rpow_zero] using h

/-- If `f` is real-valued and `x` is strictly greater than the abscissa of absolute convergence
of `f`, then the real series `∑' n, f n / n ^ x` converges. -/
lemma LSeries.summable_real_of_abscissaOfAbsConv_lt {f : ℕ → ℝ} {x : ℝ}
(h : abscissaOfAbsConv (f ·) < x) :
Summable fun n : ℕ ↦ f n / (n : ℝ) ^ x := by
have h' : abscissaOfAbsConv (f ·) < (x : ℂ).re := by simpa only [ofReal_re] using h
have := LSeriesSummable_of_abscissaOfAbsConv_lt_re h'
rw [LSeriesSummable, show term _ _ = fun n ↦ _ from rfl] at this
conv at this =>
enter [1, n]
rw [term_def, show (n : ℂ) = (n : ℝ) from rfl, ← ofReal_cpow n.cast_nonneg, ← ofReal_div,
show (0 : ℂ) = (0 : ℝ) from rfl, ← apply_ite]
rw [summable_ofReal] at this
refine this.congr_cofinite ?_
filter_upwards [Set.Finite.compl_mem_cofinite <| Set.finite_singleton 0] with n hn
simp only [Set.mem_compl_iff, Set.mem_singleton_iff] at hn
exact if_neg hn

0 comments on commit d59b190

Please sign in to comment.