Zulip Chat Archive
Stream: Is there code for X?
Topic: monotone function of iInf of antitone function
Ira Fesefeldt (Nov 25 2024 at 10:30):
I have something similar to this:
import Mathlib
variable (a : α) (b : ℕ → ℤ → α) (f : (ℤ → α) → α)
variable [CompleteLinearOrder α]
example (h_f_mono : Monotone f) (h_b_antitone : Antitone b) (h : ∀ i : ℕ, a ≤ f (fun z => b i z)) :
a ≤ f (fun z => ⨅ i, b i z) := by
sorry
Graphically this theorem looks correct to me, but I am not sure how to proof it in Lean and couldn't find any matching theorems...
Daniel Weber (Nov 25 2024 at 11:02):
I don't think this is true — f
could be a jump function, which is 0 at the infimum and 1 at any greater value. I think this is true for continuous f
, though
Ira Fesefeldt (Nov 25 2024 at 11:38):
Fair enough :/
Last updated: May 02 2025 at 03:31 UTC