Documentation

Mathlib.NumberTheory.EulerProduct.DirichletLSeries

The Euler Product for the Riemann Zeta Function and Dirichlet L-Series #

The first main result of this file is riemannZeta_eulerProduct, which states the Euler Product formula for the Riemann ζ function $$\prod_p \frac{1}{1 - p^{-s}} = \lim_{n \to \infty} \prod_{p < n} \frac{1}{1 - p^{-s}} = \zeta(s)$$ for $s$ with real part $> 1$ ($p$ runs through the primes). The formalized statement is the second equality above, since infinite products are not yet available in Mathlib.

The second result is dirichletLSeries_eulerProduct, which is the analogous statement for Dirichlet L-functions.

noncomputable def riemannZetaSummandHom {s : } (hs : s 0) :

When s ≠ 0, the map n ↦ n^(-s) is completely multiplicative and vanishes at zero.

Equations
Instances For
    noncomputable def dirichletSummandHom {s : } {n : } (χ : DirichletCharacter n) (hs : s 0) :

    When χ is a Dirichlet character and s ≠ 0, the map n ↦ χ n * n^(-s) is completely multiplicative and vanishes at zero.

    Equations
    • dirichletSummandHom χ hs = { toFun := fun (n_1 : ) => χ n_1 * n_1 ^ (-s), map_zero' := , map_one' := , map_mul' := }
    Instances For
      theorem summable_riemannZetaSummand {s : } (hs : 1 < s.re) :

      When s.re > 1, the map n ↦ n^(-s) is norm-summable.

      theorem summable_dirichletSummand {s : } {N : } (χ : DirichletCharacter N) (hs : 1 < s.re) :
      Summable fun (n : ) => (dirichletSummandHom χ ) n

      When s.re > 1, the map n ↦ χ(n) * n^(-s) is norm-summable.

      theorem riemannZeta_eulerProduct {s : } (hs : 1 < s.re) :
      Filter.Tendsto (fun (n : ) => n.primesBelow.prod fun (p : ) => (1 - p ^ (-s))⁻¹) Filter.atTop (nhds (riemannZeta s))

      The Euler product for the Riemann ζ function, valid for s.re > 1.

      theorem dirichletLSeries_eulerProduct {s : } {N : } (χ : DirichletCharacter N) (hs : 1 < s.re) :
      Filter.Tendsto (fun (n : ) => n.primesBelow.prod fun (p : ) => (1 - χ p * p ^ (-s))⁻¹) Filter.atTop (nhds (∑' (n : ), (dirichletSummandHom χ ) n))

      The Euler product for Dirichlet L-series, valid for s.re > 1.