Zulip Chat Archive
Stream: new members
Topic: Tendsto f atTop (nhds L)
Hbz (Aug 10 2025 at 14:34):
Is there a theorem in Lean4 regarding ∃ L : ℝ , Tendsto f atTop (nhds L) ↔ ∃ L, ∀ ε > 0, ∃ N, ∀ x > N, |f x - L| < ε, or a similar theorem? Or do I have to prove it manually?
Kenny Lau (Aug 10 2025 at 14:41):
@Hbz @loogle Filter.Tendsto _ Filter.atTop (nhds _) ↔ _
loogle (Aug 10 2025 at 14:41):
:search: tendsto_atTop_nhds, tendsto_const_mul_pow_nhds_iff, and 23 more
Kenny Lau (Aug 10 2025 at 14:42):
@loogle Filter.Tendsto _ Filter.atTop (nhds _) ↔ _, Norm.norm
loogle (Aug 10 2025 at 14:42):
:search: NormedAddCommGroup.tendsto_atTop, NormedAddCommGroup.tendsto_atTop', and 1 more
Matt Diamond (Aug 10 2025 at 18:56):
docs#Metric.tendsto_atTop / docs#Metric.tendsto_atTop' is close
Matt Diamond (Aug 10 2025 at 19:00):
actually I think that's exactly it
Jireh Loreaux (Aug 10 2025 at 23:55):
But to be honest, the right answer here is just to use filter bases and docs#Filter.HasBasis.tendsto_iff as the proof of the result Matt linked to does. That allows you to easily get lots of minor variations on the precise statement (e.g. if you wanted \le \eps instead at the end).
Wuyang (Aug 11 2025 at 15:59):
Looks like Metric.tendsto_atTop or its variants should match your need, and Filter.HasBasis.tendsto_iff gives flexibility for tweaks.
You can also try LeanFinder (www.leanfinder.org) to explore related limit theorems quickly.
Wuyang (Aug 11 2025 at 15:59):
@leanfinder limit theorem equivalence tendsto atTop nhds L epsilon N characterization in Lean4
leanfinder (Aug 11 2025 at 16:00):
Here’s what I found:
-
theorem tendsto_atTop' : Tendsto f atTop l ↔ ∀ s ∈ l, ∃ a, ∀ b ≥ a, f b ∈ s := by simp only [tendsto_def, mem_atTop_sets, mem_preimage] "A function tends to the filter at infinity (i.e., as ) if and only if for every set in the filter , there exists a threshold such that for all , the value belongs to ." (score: 0.744)
-
theorem Filter.tendsto_atTop' : Tendsto f atTop l ↔ ∀ s ∈ l, ∃ a, ∀ b ≥ a, f b ∈ s := by simp only [tendsto_def, mem_atTop_sets, mem_preimage] "A function tends to the filter at infinity (i.e., as ) if and only if for every set in the filter , there exists a threshold such that for all , the value belongs to ." (score: 0.744)
-
theorem Metric.tendsto_atTop [Nonempty β] [SemilatticeSup β] {u : β → α} {a : α} : Tendsto u atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n ≥ N, dist (u n) a < ε := (atTop_basis.tendsto_iff nhds_basis_ball).trans <| by simp only [true_and, mem_ball, mem_Ici] "Let be a pseudo-metric space and be a nonempty join-semilattice. For a function and a point , the function tends to as the argument tends to infinity (with respect to the order on ) if and only if for every , there exists an index such that for all , the distance ." (score: 0.736)
-
theorem tendsto_atTop [Nonempty β] [SemilatticeSup β] {u : β → α} {a : α} : Tendsto u atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n ≥ N, edist (u n) a < ε := (atTop_basis.tendsto_iff nhds_basis_eball).trans <| by simp only [exists_prop, true_and_iff, mem_Ici, mem_ball] "Let be an extended pseudo-metric space and be a nonempty join-semilattice. For a function and a point , the function tends to as approaches infinity if and only if for every , there exists such that for all , the extended distance . This means that gets arbitrarily close to as becomes large." (score: 0.734)
-
theorem Metric.tendsto_atTop' [Nonempty β] [SemilatticeSup β] [NoMaxOrder β] {u : β → α} {a : α} : Tendsto u atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n > N, dist (u n) a < ε := (atTop_basis_Ioi.tendsto_iff nhds_basis_ball).trans <| by simp only [true_and, gt_iff_lt, mem_Ioi, mem_ball] "Let be a pseudo-metric space and be a nonempty directed set (specifically, a join-semilattice) with no maximal elements. For a function and a point , the function tends to as the index tends to infinity if and only if for every , there exists an index such that for all , the distance ." (score: 0.732)
-
theorem tendsto_atTop_nhds [Nonempty α] [SemilatticeSup α] {f : α → X} : Tendsto f atTop (𝓝 x) ↔ ∀ U : Set X, x ∈ U → IsOpen U → ∃ N, ∀ n, N ≤ n → f n ∈ U := (atTop_basis.tendsto_iff (nhds_basis_opens x)).trans <| by simp only [and_imp, exists_prop, true_and, mem_Ici] "Let be a nonempty join-semilattice and a topological space. For a function , the following are equivalent:
- The function tends to the neighborhood filter along the filter
atTop(i.e., in the order topology). - For every open neighborhood of in , there exists an index such that for all , we have ." (score: 0.726)
- theorem tendsto_atTop_nhds [Nonempty α] [SemilatticeSup α] {f : α → X} : Tendsto f atTop (𝓝 x) ↔ ∀ U : Set X, x ∈ U → IsOpen U → ∃ N, ∀ n, N ≤ n → f n ∈ U := (atTop_basis.tendsto_iff (nhds_basis_opens x)).trans <| by simp only [and_imp, exists_prop, true_and, mem_Ici] "Let be a nonempty join-semilattice and a topological space. For a function , the following are equivalent:
- The function tends to the neighborhood filter along the filter
atTop(i.e., in the order topology). - For every open neighborhood of in , there exists an index such that for all , we have ." (score: 0.726)
-
theorem tendsto_atTop [Nonempty β] [SemilatticeSup β] {f : β → ℝ≥0∞} {a : ℝ≥0∞} (ha : a ≠ ∞) : Tendsto f atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n ≥ N, f n ∈ Icc (a - ε) (a + ε) := .trans (atTop_basis.tendsto_iff (hasBasis_nhds_of_ne_top ha)) (by simp only [true_and]; rfl) "Let be a nonempty join-semilattice and be a function. For any finite extended non-negative real number , the function tends to as approaches infinity if and only if for every , there exists such that for all , the value lies in the closed interval ." (score: 0.726)
-
theorem EMetric.tendsto_atTop [Nonempty β] [SemilatticeSup β] {u : β → α} {a : α} : Tendsto u atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n ≥ N, edist (u n) a < ε := (atTop_basis.tendsto_iff nhds_basis_eball).trans <| by simp only [exists_prop, true_and, mem_Ici, mem_ball] "Let be an extended pseudo-metric space and be a nonempty join-semilattice. For a function and a point , the function tends to along the filter
atTopif and only if for every , there exists such that for all , the extended distance satisfies ." (score: 0.724) -
theorem ENNReal.tendsto_atTop [Nonempty β] [SemilatticeSup β] {f : β → ℝ≥0∞} {a : ℝ≥0∞} (ha : a ≠ ∞) : Tendsto f atTop (𝓝 a) ↔ ∀ ε > 0, ∃ N, ∀ n ≥ N, f n ∈ Icc (a - ε) (a + ε) := .trans (atTop_basis.tendsto_iff (hasBasis_nhds_of_ne_top ha)) (by simp only [true_and]; rfl) "Let be a nonempty join-semilattice and be a function. For any finite extended non-negative real number , the function tends to along the filter at infinity if and only if for every , there exists such that for all , the value lies in the closed interval ." (score: 0.723)
Last updated: Dec 20 2025 at 21:32 UTC