leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: Is there code for X?

Topic: Tendsto.filter_mono


Vincent Beffara (Mar 05 2024 at 21:54):

Is there a name for this?

example {f : ℝ → ℝ} {p₁ p₂ : Filter ℝ} (h : p₁ ≤ p₂) (hf : Tendsto f p₂ (𝓝 0)) : Tendsto f p₁ (𝓝 0)

exact? tells me that it is fun _ a ↦ h (hf a), it is also map_mono h |>.trans hf but none feel right to me...

Anatole Dedecker (Mar 05 2024 at 22:08):

docs#Filter.Tendsto.mono_left ?


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll