Chebyshev functions #
This file defines the Chebyshev functions theta and psi.
These give logarithmically weighted sums of primes and prime powers.
Main definitions #
Chebyshev.psigives the sum ofArithmeticFunction.vonMangoldtChebyshev.thetagives the sum oflog pover primes
Main results #
Chebyshev.theta_eq_log_primorialshows thatθ xis the log of the product of primes up to xChebyshev.theta_le_log4_mul_xgives Chebyshev's upper bound onθChebyshev.psi_eq_sum_thetaandChebyshev.psi_eq_theta_add_sum_thetarelatepsitotheta.Chebyshev.psi_le_const_mul_selfgives Chebyshev's upper bound onψ.Chebyshev.primeCounting_eq_theta_div_log_add_integralrelates the prime counting function toθChebyshev.eventually_primeCounting_legives an upper bound on the prime counting function.
Notation #
We introduce the scoped notations θ and ψ in the Chebyshev namespace for the Chebyshev
functions.
References #
Parts of this file were upstreamed from the PrimeNumberTheoremAnd project by Kontorovich et al, https://github.com/alexKontorovich/PrimeNumberTheoremAnd.
TODOS #
- Prove Chebyshev's lower bound.
The sum of ArithmeticFunction.vonMangoldt over integers n ≤ x.
Equations
- Chebyshev.psi x = ∑ n ∈ Finset.Ioc 0 ⌊x⌋₊, ArithmeticFunction.vonMangoldt n
Instances For
The sum of ArithmeticFunction.vonMangoldt over integers n ≤ x.
Equations
- Chebyshev.termψ = Lean.ParserDescr.node `Chebyshev.termψ 1024 (Lean.ParserDescr.symbol "ψ")
Instances For
The sum of log p over primes p ≤ x.
Equations
- Chebyshev.theta x = ∑ p ∈ Finset.Ioc 0 ⌊x⌋₊ with Nat.Prime p, Real.log ↑p
Instances For
The sum of log p over primes p ≤ x.
Equations
- Chebyshev.termθ = Lean.ParserDescr.node `Chebyshev.termθ 1024 (Lean.ParserDescr.symbol "θ")
Instances For
Relating ψ and θ #
We isolate the contributions of different prime powers to ψ and use this to show that ψ and θ
are close.
A sum over prime powers may be written as a double sum over exponents and then primes.
Chebyshev's bound ψ x ≤ c x with an explicit constant.
Note that Chebyshev.psi_le gives a sharper bound with a better main term.
ψ - θ is the sum of Λ over non-primes.
Relation to prime counting #
We relate θ to the prime counting function π.
Integrability for the integral in Chebyshev.primeCounting_eq_theta_div_log_add_integral.