Eisenstein series q-expansions #
We give the q-expansion of Eisenstein series of weight k and level 1. In particular, we prove
EisensteinSeries.q_expansion_bernoulli which says that for even k with 3 ≤ k
Eisenstein series can we written as 1 - (2k / bernoulli k) ∑' n, σ_{k-1}(n) q^n where
q = exp(2πiz) and σ_{k-1}(n) is the sum of the (k-1)-th powers of the divisors of n.
We need k to be even so that the Eisenstein series are non-zero and we require k ≥ 3 so that
the series converges absolutely.
The proof relies on the identity
∑' n : ℤ, 1 / (z + n) ^ (k + 1) = ((-2πi)^(k+1) / k!) ∑' n : ℕ, n^k q^n which comes from
differentiating the expansion of π cot(πz) in terms of exponentials. Since our Eisenstein series
are defined as sums over coprime integer pairs, we also need to relate these to sums over all pairs
of integers, which is done in tsum_eisSummand_eq_riemannZeta_mul_eisensteinSeries. This then
gives the q-expansion with a Riemann zeta factor, which we simplify using the formula for
ζ(k) in terms of Bernoulli numbers to get the final result.
The infinte sum of k-th iterated derivative of the complex exponential multiplied by a
function that grows polynomially is absolutely and uniformly convergent.
This is a version of summableLocallyUniformlyOn_iteratedDerivWithin_smul_cexp for level one
and q-expansion coefficients all 1.
This is one key identity relating infinite series to q-expansions which shows that
∑' n, 1 / (z + n) ^ (k + 1) = ((-2 π I) ^ (k + 1) / k !) * ∑' n, n ^ k q ^n where
q = cexp (2 π I z).
This is a version of EisensteinSeries.qExpansion_identity for positive naturals,
which shows that ∑' n, 1 / (z + n) ^ (k + 1) = ((-2 π I) ^ (k + 1) / k !) * ∑' n : ℕ+, n ^ k q ^n
where q = cexp (2 π I z).
The q-Expansion of normalised Eisenstein series of level one with riemannZeta term.
The q-Expansion of normalised Eisenstein series of level one with bernoulli term.