Results on discretized exponentials #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We state several auxiliary results pertaining to sequences of the form ⌊c^n⌋₊
.
tendsto_div_of_monotone_of_tendsto_div_floor_pow
: If a monotone sequenceu
is such thatu ⌊c^n⌋₊ / ⌊c^n⌋₊
converges to a limitl
for allc > 1
, thenu n / n
tends tol
.sum_div_nat_floor_pow_sq_le_div_sq
: The sum of1/⌊c^i⌋₊^2
above a thresholdj
is comparable to1/j^2
, up to a multiplicative constant.
theorem
tendsto_div_of_monotone_of_exists_subseq_tendsto_div
(u : ℕ → ℝ)
(l : ℝ)
(hmono : monotone u)
(hlim : ∀ (a : ℝ), 1 < a → (∃ (c : ℕ → ℕ), (∀ᶠ (n : ℕ) in filter.at_top, ↑(c (n + 1)) ≤ a * ↑(c n)) ∧ filter.tendsto c filter.at_top filter.at_top ∧ filter.tendsto (λ (n : ℕ), u (c n) / ↑(c n)) filter.at_top (nhds l))) :
filter.tendsto (λ (n : ℕ), u n / ↑n) filter.at_top (nhds l)
If a monotone sequence u
is such that u n / n
tends to a limit l
along subsequences with
exponential growth rate arbitrarily close to 1
, then u n / n
tends to l
.
theorem
tendsto_div_of_monotone_of_tendsto_div_floor_pow
(u : ℕ → ℝ)
(l : ℝ)
(hmono : monotone u)
(c : ℕ → ℝ)
(cone : ∀ (k : ℕ), 1 < c k)
(clim : filter.tendsto c filter.at_top (nhds 1))
(hc : ∀ (k : ℕ), filter.tendsto (λ (n : ℕ), u ⌊c k ^ n⌋₊ / ↑⌊c k ^ n⌋₊) filter.at_top (nhds l)) :
filter.tendsto (λ (n : ℕ), u n / ↑n) filter.at_top (nhds l)
If a monotone sequence u
is such that u ⌊c^n⌋₊ / ⌊c^n⌋₊
converges to a limit l
for all
c > 1
, then u n / n
tends to l
. It is even enough to have the assumption for a sequence of
c
s converging to 1
.