The L-function of a Dirichlet character does not vanish on Re(s) ≥ 1 #
The main result in this file is DirichletCharacter.Lfunction_ne_zero_of_one_le_re
:
if χ
is a Dirichlet character, s ∈ ℂ
with 1 ≤ s.re
, and either χ
is nontrivial or s ≠ 1
,
then the L-function of χ
does not vanish at s
.
As a consequence, we have the corresponding statement for the Riemann ζ function:
riemannZeta_ne_zero_of_one_le_re
(which does not require s ≠ 1
, since the junk value at s = 1
happens to be non-zero).
These results are prerequisites for the Prime Number Theorem and Dirichlet's Theorem on primes in arithmetic progressions.
Outline of proofs #
We split into two cases: first, the special case of (non-trivial) quadratic characters at s = 1
;
then the remaining case when either s ≠ 1
or χ ^ 2 ≠ 1
.
The first case is handled using a positivity argument applied to the series L χ s * ζ s
: we show
that this function has non-negative Dirichlet coefficients, is strictly positive for s ≫ 0
, but
vanishes at s = -2
, so it must have a pole somewhere in between.
The second case is dealt with using the product
L(χ^0, 1 + x)^3 L(χ, 1 + x + I * y)^4 L(χ^2, 1 + x + 2 * I * y)
, which
we show has absolute value ≥ 1
for all positive x
and real y
; if L(χ, 1 + I * y) = 0
then
this product would have to tend to 0 as x → 0
, which is a contradiction.
Convolution of a Dirichlet character with ζ #
We define DirichletCharacter.zetaMul χ
to be the arithmetic function obtained by
taking the product (as arithmetic functions = Dirichlet convolution) of the
arithmetic function ζ
with χ
.
We then show that for a quadratic character χ
, this arithmetic function is multiplicative
and takes nonnegative real values.
The complex-valued arithmetic function that is the convolution of the constant
function 1
with χ
.
Equations
- χ.zetaMul = ↑ArithmeticFunction.zeta * toArithmeticFunction fun (x : ℕ) => χ ↑x
Instances For
The arithmetic function zetaMul χ
is multiplicative.
zetaMul χ
takes nonnegative real values when χ
is a quadratic character.
The logarithms of the Euler factors of a Dirichlet L-series form a summable sequence.
For positive x
and nonzero y
and a Dirichlet character χ
we have that
`|L(χ^0, 1 + x)^3 L(χ, 1 + x + I * y)^4 L(χ^2, 1 + x + 2 * I * y)| ≥ 1.
A variant of DirichletCharacter.norm_LSeries_product_ge_one
in terms of the L-functions.
If χ
is a Dirichlet character, then L(χ, s)
does not vanish when s.re = 1
except when χ
is trivial and s = 1
(then L(χ, s)
has a simple pole at s = 1
).
If χ
is a Dirichlet character, then L(χ, s)
does not vanish for s.re ≥ 1
except when χ
is trivial and s = 1
(then L(χ, s)
has a simple pole at s = 1
).
The L-function of a nontrivial Dirichlet character does not vanish at s = 1
.
The Riemann Zeta Function does not vanish on the closed half-plane re s ≥ 1
.
(Note that the value at s = 1
is a junk value, which happens to be nonzero.)