Skip to content

Commit

Permalink
feat(Topology/Order): add le_of_tendsto_of_frequently (#9583)
Browse files Browse the repository at this point in the history
Also add `ge_of_tendsto_of_frequently`
  • Loading branch information
urkud committed Jan 9, 2024
1 parent 043fa2f commit f846056
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Mathlib/Topology/Order/Basic.lean
Expand Up @@ -137,6 +137,10 @@ theorem closure_Iic (a : α) : closure (Iic a) = Iic a :=
isClosed_Iic.closure_eq
#align closure_Iic closure_Iic

theorem le_of_tendsto_of_frequently {f : β → α} {a b : α} {x : Filter β} (lim : Tendsto f x (𝓝 a))
(h : ∃ᶠ c in x, f c ≤ b) : a ≤ b :=
(isClosed_le' b).mem_of_frequently_of_tendsto h lim

theorem le_of_tendsto {f : β → α} {a b : α} {x : Filter β} [NeBot x] (lim : Tendsto f x (𝓝 a))
(h : ∀ᶠ c in x, f c ≤ b) : a ≤ b :=
(isClosed_le' b).mem_of_tendsto lim h
Expand Down Expand Up @@ -165,6 +169,10 @@ theorem closure_Ici (a : α) : closure (Ici a) = Ici a :=
isClosed_Ici.closure_eq
#align closure_Ici closure_Ici

lemma ge_of_tendsto_of_frequently {f : β → α} {a b : α} {x : Filter β} (lim : Tendsto f x (𝓝 a))
(h : ∃ᶠ c in x, b ≤ f c) : b ≤ a :=
(isClosed_ge' b).mem_of_frequently_of_tendsto h lim

theorem ge_of_tendsto {f : β → α} {a b : α} {x : Filter β} [NeBot x] (lim : Tendsto f x (𝓝 a))
(h : ∀ᶠ c in x, b ≤ f c) : b ≤ a :=
(isClosed_ge' b).mem_of_tendsto lim h
Expand Down

0 comments on commit f846056

Please sign in to comment.