Zulip Chat Archive

Stream: Is there code for X?

Topic: Inequality from eventually


Vincent Beffara (Apr 04 2024 at 18:53):

Is something like this in Mathlib? Presumably with a more elegant proof?

lemma le_of_eventually_nhdsWithin {a b : } (h : ∀ᶠ c in 𝓝[>] b, a  c) : a  b := by
  apply le_of_forall_lt' ; intro d hd
  have key : ∀ᶠ c in 𝓝[>] b, c < d := by
    apply eventually_of_mem (U := Iio d) ?_ (fun x hx => hx)
    rw [mem_nhdsWithin]
    refine Iio d, isOpen_Iio, hd, inter_subset_left _ _
  obtain x, h1, h2 := (h.and key).exists
  linarith

Anatole Dedecker (Apr 04 2024 at 19:29):

It’s probably not the easiest way, but in general all of those things can be obtained from docs#le_of_tendsto_of_tendsto


Last updated: May 02 2025 at 03:31 UTC