Documentation

Mathlib.NumberTheory.Harmonic.ZetaAsymp

Asymptotics of ζ s as s → 1 #

The goal of this file is to evaluate the limit of ζ s - 1 / (s - 1) as s → 1.

Main results #

Outline of arguments #

We consider the sum F s = ∑' n : ℕ, f (n + 1) s, where s is a real variable and f n s = ∫ x in n..(n + 1), (x - n) / x ^ (s + 1). We show that F s is continuous on [1, ∞), that F 1 = 1 - γ, and that F s = 1 / (s - 1) - ζ s / s for 1 < s.

By combining these formulae, one deduces that the limit of ζ s - 1 / (s - 1) at 𝓝[>] (1 : ℝ) exists and is equal to γ. Finally, using this and the Riemann removable singularity criterion we obtain the limit along punctured neighbourhoods of 1 in .

## Definitions

noncomputable def ZetaAsymptotics.term (n : ) (s : ) :

Auxiliary function used in studying zeta-function asymptotics.

Equations
Instances For
    noncomputable def ZetaAsymptotics.term_sum (s : ) (N : ) :

    Sum of finitely many terms.

    Equations
    Instances For
      noncomputable def ZetaAsymptotics.term_tsum (s : ) :

      Topological sum of terms.

      Equations
      Instances For
        theorem ZetaAsymptotics.term_welldef {n : } (hn : 0 < n) {s : } (hs : 0 < s) :
        IntervalIntegrable (fun (x : ) => (x - n) / x ^ (s + 1)) MeasureTheory.volume (n) (n + 1)

        Evaluation of the sum for s = 1 #

        theorem ZetaAsymptotics.term_one {n : } (hn : 0 < n) :
        ZetaAsymptotics.term n 1 = Real.log (n + 1) - Real.log n - 1 / (n + 1)

        The topological sum of ZetaAsymptotics.term (n + 1) 1 over all n : ℕ is 1 - γ. This is proved by directly evaluating the sum of the first N terms and using the limit definition of γ.

        Evaluation of the sum for 1 < s #

        theorem ZetaAsymptotics.term_of_lt {n : } (hn : 0 < n) {s : } (hs : 1 < s) :
        ZetaAsymptotics.term n s = 1 / (s - 1) * (1 / n ^ (s - 1) - 1 / (n + 1) ^ (s - 1)) - n / s * (1 / n ^ s - 1 / (n + 1) ^ s)
        theorem ZetaAsymptotics.term_sum_of_lt (N : ) {s : } (hs : 1 < s) :
        ZetaAsymptotics.term_sum s N = 1 / (s - 1) * (1 - 1 / (N + 1) ^ (s - 1)) - 1 / s * ((Finset.sum (Finset.range N) fun (n : ) => 1 / (n + 1) ^ s) - N / (N + 1) ^ s)
        theorem ZetaAsymptotics.term_tsum_of_lt {s : } (hs : 1 < s) :
        ZetaAsymptotics.term_tsum s = 1 / (s - 1) - 1 / s * ∑' (n : ), 1 / (n + 1) ^ s

        For 1 < s, the topological sum of ZetaAsymptotics.term (n + 1) s over all n : ℕ is 1 / (s - 1) - ζ s / s.

        theorem ZetaAsymptotics.zeta_limit_aux1 {s : } (hs : 1 < s) :
        ∑' (n : ), 1 / (n + 1) ^ s - 1 / (s - 1) = 1 - s * ZetaAsymptotics.term_tsum s

        Reformulation of ZetaAsymptotics.term_tsum_of_lt which is useful for some computations below.

        Continuity of the sum #

        First version of the limit formula, with a limit over real numbers tending to 1 from above.

        The function ζ s - 1 / (s - 1) tends to γ as s → 1.

        theorem isBigO_riemannZeta_sub_one_div {F : Type u_1} [Norm F] [One F] [NormOneClass F] :
        (fun (s : ) => riemannZeta s - 1 / (s - 1)) =O[nhds 1] fun (x : ) => 1