Zulip Chat Archive

Stream: Is there code for X?

Topic: Shifted limits


Michael Stoll (Dec 19 2023 at 22:23):

I'm looking for something like

import Mathlib

example (f : โ„‚ โ†’ โ„‚) : Tendsto f (๐“[โ‰ ] 1) (๐“ 1) โ†” Tendsto (fun z โ†ฆ f (1 + z)) (๐“[โ‰ ] 0) (๐“ 1) := by
  sorry

but have difficulties finding it.

Jireh Loreaux (Dec 19 2023 at 22:28):

Isn't this just an application of docs#Filter.Tendsto.comp ?

Michael Stoll (Dec 19 2023 at 22:29):

I guess so. I think I was looking for something involving comp, but may have mistyped (it is getting late ...).

Michael Stoll (Dec 19 2023 at 22:37):

Is there a tactic that clears Tendsto (fun x โ†ฆ 1 - x) (๐“[โ‰ ] 1) (๐“[โ‰ ] 0)?

Jireh Loreaux (Dec 19 2023 at 23:06):

Hmm... perhaps I led you astray. This works though:

import Mathlib

open Topology Filter

example (f : โ„‚ โ†’ โ„‚) : Tendsto f (๐“[โ‰ ] 1) (๐“ 1) โ†” Tendsto (fun z โ†ฆ f (1 + z)) (๐“[โ‰ ] 0) (๐“ 1) := by
  rw [โ† Function.comp, โ† tendsto_map'_iff]
  congr!
  simpa using (Homeomorph.addLeft (1 : โ„‚)).toPartialHomeomorph.map_nhdsWithin_eq
    (Set.mem_univ 0) ({0}แถœ) |>.symm

The first two lines get it down to the essence of the argument.

Patrick Massot (Dec 19 2023 at 23:22):

That toPartialHomeomorph.map_nhdsWithin_eq is really ugly. If the lemma is missing for homeomorphisms then it should be added.

Jireh Loreaux (Dec 19 2023 at 23:56):

Indeed, I think it's missing. If I can get to it, I'll PR, but i'm quite busy at the moment.

Jireh Loreaux (Dec 19 2023 at 23:59):

I guess we have docs#Set.LeftInvOn.map_nhdsWithin_eq, but that's not really better.

Jireh Loreaux (Dec 20 2023 at 00:04):

Oh, I guess we have docs#Embedding.map_nhdsWithin_eq. So the above can be written:

import Mathlib

open Topology Filter

example (f : โ„‚ โ†’ โ„‚) : Tendsto f (๐“[โ‰ ] 1) (๐“ 1) โ†” Tendsto (fun z โ†ฆ f (1 + z)) (๐“[โ‰ ] 0) (๐“ 1) := by
  rw [โ† Function.comp, โ† tendsto_map'_iff]
  congr!
  simpa using (Homeomorph.addLeft (1 : โ„‚)).embedding.map_nhdsWithin_eq ({0}แถœ) 0 |>.symm

which I think is fine.


Last updated: Dec 20 2023 at 11:08 UTC