Commit 2025-01-27 10:18 c33fe046
View on Github →feat(NumberTheory/LSeries): results involving partial sums of coefficients (part 1) (#20661) We prove several results involving partial sums of coefficients (or norm of coefficients) of L-series. The two main results of this PR are:
LSeriesSummable_of_sum_norm_bigO
: forf : ℕ → ℂ
, if the partial sums∑ k ∈ Icc 1 n, ‖f k‖
areO(n ^ r)
for some real0 ≤ r
, then the L-seriesLseries f
converges ats : ℂ
for alls
such thatr < s.re
.LSeries_eq_mul_integral
: forf : ℕ → ℂ
, if the partial sums∑ k ∈ Icc 1 n, f k
areO(n ^ r)
for some real0 ≤ r
and the L-seriesLSeries f
converges ats : ℂ
withr < s.re
, thenLSeries f s = s * ∫ t in Set.Ioi 1, (∑ k ∈ Icc 1 ⌊t⌋₊, f k) * t ^ (- (s + 1))
. More results will be proved in #20660