Zulip Chat Archive
Stream: Is there code for X?
Topic: ContinuousAt iff Tendsto on a punctured nhd
Geoffrey Irving (Oct 24 2024 at 20:36):
I feel like we have to have this, but I can't find it:
lemma continuousAt_iff_tendsto_nhdsWithin {X Y : Type} [TopologicalSpace X] [TopologicalSpace Y]
{f : X โ Y} {x : X} : ContinuousAt f x โ Tendsto f (๐[โ ] x) (๐ (f x)) := by
constructor
ยท exact tendsto_nhdsWithin_of_tendsto_nhds
ยท intro h
simp only [ContinuousAt, โ nhdsWithin_compl_singleton_sup_pure x]
exact h.sup (tendsto_pure_nhds f x)
Geoffrey Irving (Oct 24 2024 at 20:37):
To add to the frustration, I seem to remember proving this before myself, but I can't find that either.
Geoffrey Irving (Oct 24 2024 at 20:38):
Aha, found what I needed: docs#nhdsWithin_compl_singleton_sup_pure.
Yury G. Kudryashov (Oct 29 2024 at 20:32):
See docs#continuousWithinAt_compl_self
Last updated: May 02 2025 at 03:31 UTC