Convergence of p
-series #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove that the series ∑' k in ℕ, 1 / k ^ p
converges if and only if p > 1
.
The proof is based on the
Cauchy condensation test: ∑ k, f k
converges if and only if so does ∑ k, 2 ^ k f (2 ^ k)
. We prove this test in
nnreal.summable_condensed_iff
and summable_condensed_iff_of_nonneg
, then use it to prove
summable_one_div_rpow
. After this transformation, a p
-series turns into a geometric series.
TODO #
It should be easy to generalize arguments to Schlömilch's generalization of the Cauchy condensation test once we need it.
Tags #
p-series, Cauchy condensation test
Cauchy condensation test #
In this section we prove the Cauchy condensation test: for f : ℕ → ℝ≥0
or f : ℕ → ℝ
,
∑ k, f k
converges if and only if so does ∑ k, 2 ^ k f (2 ^ k)
. Instead of giving a monolithic
proof, we split it into a series of lemmas with explicit estimates of partial sums of each series in
terms of the partial sums of the other series.
Convergence of the p
-series #
In this section we prove that for a real number p
, the series ∑' n : ℕ, 1 / (n ^ p)
converges if
and only if 1 < p
. There are many different proofs of this fact. The proof in this file uses the
Cauchy condensation test we formalized above. This test implies that ∑ n, 1 / (n ^ p)
converges if
and only if ∑ n, 2 ^ n / ((2 ^ n) ^ p)
converges, and the latter series is a geometric series with
common ratio 2 ^ {1 - p}
.
Divergence of the Harmonic Series