Zulip Chat Archive

Stream: Is there code for X?

Topic: filter tendsto limit from left right top bottom


rtertr (Sonia) (May 26 2023 at 18:11):

Hello! (Sorry for the bad title, just wanted the post to be found by the most people who could need it)

I want to use tendsto_nhds_unique: tendsto f l (nhds a) → tendsto f l (nhds b) → a = b where the filter l should be x -> 0+.
I haven't been able to find any lemmas about taking the limit from above/below. Is there any tendsto theorems like that somewhere? :)

Kind regards,

Patrick Massot (May 26 2023 at 18:21):

You should look at the list of variations on neighborhood filters at https://leanprover-community.github.io/mathlib_docs/topology/basic.html#notation

Patrick Massot (May 26 2023 at 18:22):

The one you want is 𝓝[>] 0.

Patrick Massot (May 26 2023 at 18:24):

import topology.instances.real

open filter
open_locale topology

example {X : Type*} [topological_space X] [t2_space X] {f :   X} {a b}
  (ha : tendsto f (𝓝[>] 0) (𝓝 a)) (hb : tendsto f (𝓝[>] 0) (𝓝 b)) : a = b :=
tendsto_nhds_unique ha hb

rtertr (Sonia) (May 26 2023 at 18:32):

Ah, great! Thank you :D


Last updated: Dec 20 2023 at 11:08 UTC