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 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). riemannZeta_eulerProduct is the second equality above. There are versions riemannZeta_eulerProduct_hasProd and riemannZeta_eulerProduct_tprod in terms of HasProd and tprod, respectively.

The second result is dirichletLSeries_eulerProduct (with variants dirichletLSeries_eulerProduct_hasProd and dirichletLSeries_eulerProduct_tprod), which is the analogous statement for Dirichlet L-series.

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 tsum_riemannZetaSummand {s : } (hs : 1 < s.re) :
      ∑' (n : ), (riemannZetaSummandHom ) n = riemannZeta s
      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 tsum_dirichletSummand {s : } {N : } (χ : DirichletCharacter N) (hs : 1 < s.re) :
      ∑' (n : ), (dirichletSummandHom χ ) n = LSeries (fun (n : ) => χ n) s
      theorem riemannZeta_eulerProduct_hasProd {s : } (hs : 1 < s.re) :
      HasProd (fun (p : Nat.Primes) => (1 - p ^ (-s))⁻¹) (riemannZeta s)

      The Euler product for the Riemann ζ function, valid for s.re > 1. This version is stated in terms of HasProd.

      theorem riemannZeta_eulerProduct_tprod {s : } (hs : 1 < s.re) :
      ∏' (p : Nat.Primes), (1 - p ^ (-s))⁻¹ = riemannZeta s

      The Euler product for the Riemann ζ function, valid for s.re > 1. This version is stated in terms of tprod.

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

      The Euler product for the Riemann ζ function, valid for s.re > 1. This version is stated in the form of convergence of finite partial products.

      theorem dirichletLSeries_eulerProduct_hasProd {s : } {N : } (χ : DirichletCharacter N) (hs : 1 < s.re) :
      HasProd (fun (p : Nat.Primes) => (1 - χ p * p ^ (-s))⁻¹) (LSeries (fun (n : ) => χ n) s)

      The Euler product for Dirichlet L-series, valid for s.re > 1. This version is stated in terms of HasProd.

      theorem dirichletLSeries_eulerProduct_tprod {s : } {N : } (χ : DirichletCharacter N) (hs : 1 < s.re) :
      ∏' (p : Nat.Primes), (1 - χ p * p ^ (-s))⁻¹ = LSeries (fun (n : ) => χ n) s

      The Euler product for Dirichlet L-series, valid for s.re > 1. This version is stated in terms of tprod.

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

      The Euler product for Dirichlet L-series, valid for s.re > 1. This version is stated in the form of convergence of finite partial products.