leanprover-community / mathport

Mathport is a tool for porting Lean3 projects to Lean4
Apache License 2.0
41 stars 15 forks source link

`theorem _root_` #131

Closed gebner closed 2 years ago

gebner commented 2 years ago
theorem _root_.continuous.exists_forall_le [Nonempty β] {f : β → α} (hf : Continuous f)
    (hlim : Tendsto f (cocompact β) atTop) : ∃ x, ∀ y, f x ≤ f y := by
gebner commented 2 years ago

This is implemented upstream now: https://github.com/leanprover/lean4/issues/490