Documentation

Mathlib.NumberTheory.LSeries.HurwitzZetaEven

Even Hurwitz zeta functions #

In this file we study the functions on which are the meromorphic continuation of the following series (convergent for 1 < re s), where a ∈ ℝ is a parameter:

completedHurwitzZetaEven a s = 1 / 2 * □ * ∑' n : ℤ, 1 / |n + a| ^ s

and

completedCosZeta a s = □ * ∑' n : ℕ, cos (2 * π * a * n) / |n| ^ s

where denotes a Gamma factor. Note that the term for n = -a in the first sum is omitted if a is an integer, and the term for n = 0 is omitted in the second sum (always).

Of course, we cannot define these functions by the above formulae (since existence of the meromorphic continuation is not at all obvious); we in fact construct them as Mellin transforms of various versions of the Jacobi theta function. We also define modified versions with a subscript 0 which are entire functions differing from the above by multiples of 1 / s and 1 / (1 - s).

## Main definitions and theorems

Definitions and elementary properties of kernels #

@[irreducible]
def evenKernel (a : UnitAddCircle) (x : ) :

Even Hurwitz zeta kernel (function whose Mellin transform will be the even part of the completed Hurwit zeta function). See evenKernel_def for the defining formula, and hasSum_int_evenKernel for an expression as a sum over .

Equations
Instances For
    theorem evenKernel_def (a : ) (x : ) :
    (evenKernel (a) x) = Complex.exp (-Real.pi * a ^ 2 * x) * jacobiTheta₂ (a * Complex.I * x) (Complex.I * x)
    theorem evenKernel_undef (a : UnitAddCircle) {x : } (hx : x 0) :

    For x ≤ 0 the defining sum diverges, so the kernel is 0.

    @[irreducible]
    def cosKernel (a : UnitAddCircle) (x : ) :

    Cosine Hurwitz zeta kernel. See cosKernel_def for the defining formula, and hasSum_int_cosKernel for expression as a sum.

    Equations
    Instances For
      theorem cosKernel_def (a : ) (x : ) :
      (cosKernel (a) x) = jacobiTheta₂ (a) (Complex.I * x)
      theorem cosKernel_undef (a : UnitAddCircle) {x : } (hx : x 0) :
      cosKernel a x = 0

      For a = 0, both kernels agree.

      theorem evenKernel_functional_equation (a : UnitAddCircle) (x : ) :
      evenKernel a x = 1 / x ^ (1 / 2) * cosKernel a (1 / x)

      Formulae for the kernels as sums #

      theorem hasSum_int_evenKernel (a : ) {t : } (ht : 0 < t) :
      HasSum (fun (n : ) => Real.exp (-Real.pi * (n + a) ^ 2 * t)) (evenKernel (a) t)
      theorem hasSum_int_cosKernel (a : ) {t : } (ht : 0 < t) :
      HasSum (fun (n : ) => Complex.exp (2 * Real.pi * Complex.I * a * n) * (Real.exp (-Real.pi * n ^ 2 * t))) (cosKernel (a) t)
      theorem hasSum_int_evenKernel₀ (a : ) {t : } (ht : 0 < t) :
      HasSum (fun (n : ) => if n + a = 0 then 0 else Real.exp (-Real.pi * (n + a) ^ 2 * t)) (evenKernel (a) t - if a = 0 then 1 else 0)

      Modified version of hasSum_int_evenKernel omitting the constant term at .

      theorem hasSum_int_cosKernel₀ (a : ) {t : } (ht : 0 < t) :
      HasSum (fun (n : ) => if n = 0 then 0 else Complex.exp (2 * Real.pi * Complex.I * a * n) * (Real.exp (-Real.pi * n ^ 2 * t))) ((cosKernel (a) t) - 1)
      theorem hasSum_nat_cosKernel₀ (a : ) {t : } (ht : 0 < t) :
      HasSum (fun (n : ) => 2 * Real.cos (2 * Real.pi * a * (n + 1)) * Real.exp (-Real.pi * (n + 1) ^ 2 * t)) (cosKernel (a) t - 1)

      Asymptotics of the kernels as t → ∞ #

      theorem isBigO_atTop_evenKernel_sub (a : UnitAddCircle) :
      ∃ (p : ), 0 < p (fun (x : ) => evenKernel a x - if a = 0 then 1 else 0) =O[Filter.atTop] fun (x : ) => Real.exp (-p * x)

      The function evenKernel a - L has exponential decay at +∞, where L = 1 if a = 0 and L = 0 otherwise.

      theorem isBigO_atTop_cosKernel_sub (a : UnitAddCircle) :
      ∃ (p : ), 0 < p (fun (x : ) => cosKernel a x - 1) =O[Filter.atTop] fun (x : ) => Real.exp (-p * x)

      The function cosKernel a - 1 has exponential decay at +∞, for any a.

      Construction of a FE-pair #

      A WeakFEPair structure with f = evenKernel a and g = cosKernel a.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        Definition of the completed even Hurwitz zeta function #

        The meromorphic function of s which agrees with 1 / 2 * Gamma (s / 2) * π ^ (-s / 2) * ∑' (n : ℤ), 1 / |n + a| ^ s for 1 < re s.

        Equations
        Instances For

          The entire function differing from completedHurwitzZetaEven a s by a linear combination of 1 / s and 1 / (1 - s).

          Equations
          Instances For
            theorem completedHurwitzZetaEven_eq (a : UnitAddCircle) (s : ) :
            completedHurwitzZetaEven a s = completedHurwitzZetaEven₀ a s - (if a = 0 then 1 else 0) / s - 1 / (1 - s)

            The meromorphic function of s which agrees with Gamma (s / 2) * π ^ (-s / 2) * ∑' n : ℕ, cos (2 * π * a * n) / n ^ s for 1 < re s.

            Equations
            Instances For

              The entire function differing from completedCosZeta a s by a linear combination of 1 / s and 1 / (1 - s).

              Equations
              Instances For
                theorem completedCosZeta_eq (a : UnitAddCircle) (s : ) :
                completedCosZeta a s = completedCosZeta₀ a s - 1 / s - (if a = 0 then 1 else 0) / (1 - s)

                Parity and functional equations #

                Functional equation for the even Hurwitz zeta function.

                Functional equation for the even Hurwitz zeta function with poles removed.

                Functional equation for the even Hurwitz zeta function (alternative form).

                Functional equation for the even Hurwitz zeta function with poles removed (alternative form).