We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent e4bb754 commit 3f8d2b6Copy full SHA for 3f8d2b6
Mathlib/Order/Filter/Extr.lean
@@ -195,6 +195,12 @@ theorem isMaxOn_const {b : β} : IsMaxOn (fun _ => b) s a :=
195
theorem isExtrOn_const {b : β} : IsExtrOn (fun _ => b) s a :=
196
isExtrFilter_const
197
198
+/-- If `f` has a minimum and a maximum both given by `f a` along the filter `l`, then it is
199
+eventually equal to `f a` along the filter. -/
200
+lemma eventuallyEq_of_isMinFilter_of_isMaxFilter {β : Type*} [PartialOrder β] {f : α → β}
201
+ (h₁ : IsMinFilter f l a) (h₂ : IsMaxFilter f l a) : f =ᶠ[l] (fun _ ↦ f a) := by
202
+ filter_upwards [h₁, h₂] using by grind
203
+
204
/-! ### Order dual -/
205
206
0 commit comments