Zulip Chat Archive
Stream: Is there code for X?
Topic: Limit on neighborhood from punctured neighborhood
Michael Stoll (Jan 02 2024 at 19:23):
How to prove the following?
import Mathlib
open Filter Topology in
example (f : ℂ → ℂ) (w z : ℂ) (h₁ : Tendsto f (𝓝[≠] w) (𝓝 z)) (h₂ : f w = z) :
Tendsto f (𝓝 w) (𝓝 z) := by sorry
Michael Stoll (Jan 02 2024 at 19:23):
@loogle (Filter.Tendsto ?f (nhdsWithin ?w ?_) (nhds ?z)), (Filter.Tendsto ?f (nhds ?w) (nhds ?z))
loogle (Jan 02 2024 at 19:23):
:shrug: nothing found
Yaël Dillies (Jan 02 2024 at 19:24):
Why not just rewrite h₂
?
Michael Stoll (Jan 02 2024 at 19:28):
So, how to prove
import Mathlib
open Filter Topology in
example (f : ℂ → ℂ) (w : ℂ) (h₁ : Tendsto f (𝓝[≠] w) (𝓝 (f w))) :
Tendsto f (𝓝 w) (𝓝 (f w)) := by sorry
then? (Still no match in Loogle.)
Michael Stoll (Jan 02 2024 at 19:29):
Ah: docs#continuousWithinAt_compl_self .
Michael Stoll (Jan 02 2024 at 19:29):
Need to write this as a continuity statement (which is what I came from originally).
Anatole Dedecker (Jan 02 2024 at 19:46):
You can also rewrite using docs#nhdsWithin_compl_singleton_sup_pure and docs#Filter.tendsto_sup, and then use docs#tendsto_pure_nhds
Last updated: May 02 2025 at 03:31 UTC