Zulip Chat Archive
Stream: Is there code for X?
Topic: Shift pointed neighborhoods?
Michael Stoll (Jan 14 2024 at 14:21):
I'm looking for the following:
import Mathlib
open Topology
example : Filter.Tendsto (fun w : โ โฆ 1 + w) (๐[โ ] 0) (๐[โ ] 1) := by
sorry
There are lemmas like docs#Filter.Tendsto.const_add, but they seem to always need a non-pointed neighborhood in the target. I tried to fiddle around a bit with apply?
, but it did not seem to produce anything helpful.
@loogle Filter.Tendsto, "const", "add"
loogle (Jan 14 2024 at 14:21):
:search: Filter.tendsto_atBot_add_const_left, Filter.tendsto_atBot_add_const_right, and 11 more
Michael Stoll (Jan 14 2024 at 14:23):
example : Filter.Tendsto (fun w : โ โฆ 1 + w) (๐[โ ] 0) (๐[โ ] 1) := by
refine Filter.tendsto_iff_comap.mpr <| Eq.le ?_
leaves me at โข ๐[โ ] 0 = Filter.comap (fun w โฆ 1 + w) (๐[โ ] 1)
, which looks like simp
or so should be able to solve it, but no luck...
Anatole Dedecker (Jan 14 2024 at 14:39):
I would try to use docs#tendsto_nhdsWithin_iff together with docs#eventually_nhdsWithin_of_forall
Anatole Dedecker (Jan 14 2024 at 14:41):
Or use the fact that your map is an homeomorphism and docs#Embedding.map_nhdsWithin_eq
Anatole Dedecker (Jan 14 2024 at 14:42):
But I guess some more specialized API for the case of homeomorphisms wouldnโt hurt
Michael Stoll (Jan 14 2024 at 15:05):
This comes up when you want to change the base-point of a limit, as in
open Topology Filter
example (f : โ โ โ) (a b c : โ) :
Tendsto (fun z โฆ f (a + z)) (๐[โ ] b) (๐ c) โ Tendsto f (๐[โ ] (a + b)) (๐ c) := sorry
It would be nice to have lemmas in Mathlib that make that easy.
Michael Stoll (Jan 14 2024 at 15:21):
To un-#xy, this is what I'm really after here:
import Mathlib
open Topology Filter
example {f : โ โ โ} (h : Tendsto (fun z โฆ (z - 1) * f z) (๐[โ ] 1) (๐ 1)) :
(fun w โฆ f (1 + w)) =O[๐[โ ] 1] (โ.โโปยน) := by
sorry
Maybe the approach I was taking is not the best one?
Patrick Massot (Jan 14 2024 at 15:24):
Didn't we have the exact same conversation a couple of weeks ago?
Patrick Massot (Jan 14 2024 at 15:25):
Michael Stoll (Jan 14 2024 at 15:28):
Right (I had forgotten about that conversation). I guess the lemmas you were suggesting there are still missing. So I'll try to open a PR adding them. Re-reading, I see that you did open #9166, but it has not been merged so far.
Michael Stoll (Jan 14 2024 at 15:30):
It is labeled "awaiting-author" since three weeks or so...
Patrick Massot (Jan 14 2024 at 15:32):
Ok, I commited the suggested change, let's see if it builds.
Michael Stoll (Jan 14 2024 at 15:51):
Is there an easy way of constructing the homeomorphism given by translation (on a topological (additive) group)?
Yaรซl Dillies (Jan 14 2024 at 15:52):
Michael Stoll (Jan 14 2024 at 15:54):
(I needed docs#Homeomorph.addLeft instead.)
Last updated: May 02 2025 at 03:31 UTC