Zulip Chat Archive

Stream: Is there code for X?

Topic: Bijections and Inverses, Cauchy sequence permutations


Yury G. Kudryashov (Feb 12 2022 at 01:10):

We have docs#filter.tendsto.comp

Yury G. Kudryashov (Feb 12 2022 at 01:12):

So you have

example {α : Type*} [topological_space α] {u :   α} {a : α} (hu : tendsto u at_top (𝓝 a))
  {f :   } (hf : function.injective f) : tendsto (u  f) at_top (𝓝 a) :=
hu.comp hf.tendsto_at_top

Yury G. Kudryashov (Feb 12 2022 at 01:13):

I don't think that we should add this as a separate lemma.

Kevin Buzzard (Feb 12 2022 at 10:04):

@Mark Gerads what's going on here is that the lemma you're proving is just the sort of thing which we see in undergraduate analysis textbooks, but in fact it's an easy consequence of a far more general lemma about filters on uniform spaces and mathlib is focused on proving things in this kind of large generality. Mathlib is not designed for pedagogy, it is like Bourbaki, striving for maximal generality rather than concrete examples such as your application

Kevin Buzzard (Feb 12 2022 at 10:07):

The very fact that you want to state the lemma for both real and complex sequences is exactly the reason we state it for neither. Next week someone will want it for sequences of p-adic numbers, the week after someone will want it for ℝ^3 etc

Mark Gerads (Feb 12 2022 at 20:55):

Oh, I definitely support having every proof as general as possible. I am glad that [a much more general proof than what I had in mind] was submitted to mathlib.


Last updated: Dec 20 2023 at 11:08 UTC