A collection of specific limit computations #
This file, by design, is independent of NormedSpace in the import hierarchy. It contains
important specific limit computations in metric spaces, in ordered rings/fields, and in specific
instances of these such as ℝ, ℝ≥0 and ℝ≥0∞.
The limit of n / (n + x) is 1, for any constant x (valid in ℝ or any topological division
algebra over ℚ≥0, e.g., ℂ).
For any positive m : ℕ, ((n % m : ℕ) : ℝ) / (n : ℝ) tends to 0 as n tends to ∞.
If a ≠ 0, (a * x + c)⁻¹ tends to 0 as x tends to ∞.
If g tends to ∞, then eventually for all x we have (f x / g x) * g x = f x.
If when x tends to ∞, g tends to ∞ and f x / g x tends to a positive
constant, then f tends to ∞.
If when x tends to ∞, g tends to ∞ and f x / g x tends to a positive
constant, then f tends to ∞.
If when x tends to ∞, f x / g x tends to a positive constant, then f tends to ∞ if
and only if g tends to ∞.
Powers #
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.
Summability tests based on comparison with geometric series #
Positive sequences with small sums on countable types #
For any positive ε, define on an encodable type a positive sequence with sum less than ε
Equations
- posSumOfEncodable hε ι = ⟨(fun (n : ℕ) => ε / 2 / 2 ^ n) ∘ Encodable.encode, ⋯⟩
Instances For
Factorial #
Ceil and floor #
Alias of tendsto_inv_atTop_nhds_zero_nat.
Alias of tendsto_inv_atTop_nhds_zero_nat.
Alias of tendsto_const_div_atTop_nhds_zero_nat.
Alias of tendsto_pow_atTop_atTop_of_one_lt.