Zulip Chat Archive

Stream: mathlib4

Topic: limits of functions defined on subset of domain


Amos Turchet (Aug 05 2024 at 12:52):

In PR #14442 we needed some lemmas about limits of functions f: ℕ → ℝ that coincided with functions g: ℝ → ℝ for which the same limit was already in mathlib.

Example:

lemma tendsto_nat_rpow_div : Filter.Tendsto (fun k :   (k : ) ^ (k : )⁻¹)
     Filter.atTop (nhds 1) :=

This existed already for real-valued functions with domain .

In the original PR we inserted these auxiliary lemmas, proved by hand, but it seems that a more general statement might/should be in Mathlib. Since the PR is still under review we (with @Fabrizio Barroero ) proposed a couple of more general statements like:

theorem aux {l: Filter } {f :   } {g:   } (hg: ∀ᶠ n in atTop, g n = f n)
     (hl : Filter.Tendsto f Filter.atTop l) : Filter.Tendsto g Filter.atTop l

or even more generally

theorem aux' {α : Type*} [Nonempty α] [LinearOrder α] {l : Filter } {f :   } {g : α  }
    {c : α  } (hc₀ : Monotone c) (hc :  x : ,  a : α, x  c a)
    (hg : ∀ᶠ n in atTop, g n = f (c n)) (hl : Filter.Tendsto f Filter.atTop l) :
    Filter.Tendsto g Filter.atTop l

I guess one could keep generalizing this to arbitrary functions sharing an accumulation point and coinciding eventually at a filter, but we are unsure what is the best way to procede.

Shall we stick with what is needed for our PR (that is about Ostrowski theorem), i.e. the specific lemmas? Or rather try to write some more general statement that works for real-valued functions, like the theorems above? Or even wait for some topology experts to formulate the most general statement?

Etienne Marion (Aug 05 2024 at 13:07):

I’m definitely not an expert, but isn’t this just a composition of limit, because the coercion from Nat to Real tends to atTop along atTop?

Etienne Marion (Aug 05 2024 at 13:07):

docs#tendsto_natCast_atTop_atTop


Last updated: May 02 2025 at 03:31 UTC