A collection of specific limit computations #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains important specific limit computations in (semi-)normed groups/rings/spaces, as
as well as such computations in ℝ
when the natural proof passes through a fact about normed
spaces.
Powers #
The (scalar) product of a sequence that tends to zero with a bounded one also tends to zero.
Various statements equivalent to the fact that f n
grows exponentially slower than R ^ n
.
- 0: $f n = o(a ^ n)$ for some $-R < a < R$;
- 1: $f n = o(a ^ n)$ for some $0 < a < R$;
- 2: $f n = O(a ^ n)$ for some $-R < a < R$;
- 3: $f n = O(a ^ n)$ for some $0 < a < R$;
- 4: there exist
a < R
andC
such that one ofC
andR
is positive and $|f n| ≤ Ca^n$ for alln
; - 5: there exists
0 < a < R
and a positiveC
such that $|f n| ≤ Ca^n$ for alln
; - 6: there exists
a < R
such that $|f n| ≤ a ^ n$ for sufficiently largen
; - 7: there exists
0 < a < R
such that $|f n| ≤ a ^ n$ for sufficiently largen
.
NB: For backwards compatibility, if you add more items to the list, please append them at the end of the list.
For any natural k
and a real r > 1
we have n ^ k = o(r ^ n)
as n → ∞
.
For a real r > 1
we have n = o(r ^ n)
as n → ∞
.
If |r| < 1
, then n ^ k r ^ n
tends to zero for any natural k
.
If 0 ≤ r < 1
, then n ^ k r ^ n
tends to zero for any natural k
.
This is a specialized version of tendsto_pow_const_mul_const_pow_of_abs_lt_one
, singled out
for ease of application.
If |r| < 1
, then n * r ^ n
tends to zero.
If 0 ≤ r < 1
, then n * r ^ n
tends to zero. This is a specialized version of
tendsto_self_mul_const_pow_of_abs_lt_one
, singled out for ease of application.
In a normed ring, the powers of an element x with ‖x‖ < 1
tend to zero.
Geometric series #
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
.
Summability tests based on comparison with geometric series #
Dirichlet and alternating series tests #
Dirichlet's Test for monotone sequences.
Dirichlet's test for antitone sequences.
The alternating series test for monotone sequences.
See also tendsto_alternating_series_of_monotone_tendsto_zero
.
The alternating series test for monotone sequences.
The alternating series test for antitone sequences.
See also tendsto_alternating_series_of_antitone_tendsto_zero
.
The alternating series test for antitone sequences.
Factorial #
The series ∑' n, x ^ n / n!
is summable of any x : ℝ
. See also exp_series_div_summable
for a version that also works in ℂ
, and exp_series_summable'
for a version that works in
any normed algebra over ℝ
or ℂ
.