Zulip Chat Archive
Stream: general
Topic: monotonicity lemma
Rob Lewis (Sep 28 2018 at 13:00):
I feel like this lemma (or similar) must exist somewhere already, but I'm coming up empty -- anyone recognize this?
example {α} [partial_order α] (f : ℕ → α) (h : ∀ n, f (n+1) ≤ f n) : ∀ m n, m ≤ n → f n ≤ f m
Last updated: May 02 2025 at 03:31 UTC