A collection of specific limit computations
Powers
In a normed ring, the powers of an element x with ∥x∥ < 1
tend to zero.
Geometric series
Sequences with geometrically decaying distance in metric spaces
In this paragraph, we discuss sequences in metric spaces or emetric spaces for which the distance between two consecutive terms decays geometrically. We show that such sequences are Cauchy sequences, and bound their distances to the limit. We also discuss series with geometrically decaying terms.
If edist (f n) (f (n+1))
is bounded by C * r^n
, then the distance from
f n
to the limit of f
is bounded above by C * r^n / (1 - r)
.
If edist (f n) (f (n+1))
is bounded by C * r^n
, then the distance from
f 0
to the limit of f
is bounded above by C / (1 - r)
.
If edist (f n) (f (n+1))
is bounded by C * 2^-n
, then the distance from
f n
to the limit of f
is bounded above by 2 * C * 2^-n
.
If edist (f n) (f (n+1))
is bounded by C * 2^-n
, then the distance from
f 0
to the limit of f
is bounded above by 2 * C
.
If dist (f n) (f (n+1))
is bounded by C * r^n
, r < 1
, then the distance from
f n
to the limit of f
is bounded above by C * r^n / (1 - r)
.
If dist (f n) (f (n+1))
is bounded by C * r^n
, r < 1
, then the distance from
f 0
to the limit of f
is bounded above by C / (1 - r)
.
If dist (f n) (f (n+1))
is bounded by (C / 2) / 2^n
, then the distance from
f 0
to the limit of f
is bounded above by C
.
If dist (f n) (f (n+1))
is bounded by (C / 2) / 2^n
, then the distance from
f n
to the limit of f
is bounded above by C / 2^n
.
If ∥f n∥ ≤ C * r ^ n
for all n : ℕ
and some r < 1
, then the partial sums of f
form a
Cauchy sequence. This lemma does not assume 0 ≤ r
or 0 ≤ C
.
If ∥f n∥ ≤ C * r ^ n
for all n : ℕ
and some r < 1
, then the partial sums of f
are within
distance C * r ^ n / (1 - r)
of the sum of the series. This lemma does not assume 0 ≤ r
or
0 ≤ C
.
A geometric series in a complete normed ring is summable. Proved above (same name, different namespace) for not-necessarily-complete normed fields.
Bound for the sum of a geometric series in a normed ring. This formula does not assume that the
normed ring satisfies the axiom ∥1∥ = 1
.
Positive sequences with small sums on encodable types
For any positive ε
, define on an encodable type a positive sequence with sum less than ε
Harmonic series
Here we define the harmonic series and prove some basic lemmas about it, leading to a proof of its divergence to +∞
The harmonic series 1 + 1/2 + 1/3 + ... + 1/n
Equations
- harmonic_series n = ∑ (i : ℕ) in finset.range n, 1 / (↑i + 1)
The harmonic series diverges to +∞