Lemmas on infinite sums over the antidiagonal of the divisors function #
This file contains lemmas about the antidiagonal of the divisors function. It defines the map from
Nat.divisorsAntidiagonal n
to ℕ+ × ℕ+
given by sending n = a * b
to (a, b)
.
We then prove some identities about the infinite sums over this antidiagonal, such as
∑' n : ℕ+, n ^ k * r ^ n / (1 - r ^ n) = ∑' n : ℕ+, σ k n * r ^ n
which are used for Eisenstein series and their q-expansions. This is also a special case of
Lambert series.
The equivalence from the union over n
of Nat.divisorsAntidiagonal n
to ℕ+ × ℕ+
given by sending n = a * b
to (a, b)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
summable_prod_mul_pow
{𝕜 : Type u_1}
[NontriviallyNormedField 𝕜]
[CompleteSpace 𝕜]
[NormSMulClass ℤ 𝕜]
(k : ℕ)
{r : 𝕜}
(hr : ‖r‖ < 1)
: