Zulip Chat Archive
Stream: general
Topic: monotone
Kenny Lau (Mar 29 2018 at 08:01):
sehr geehrter @Johannes Hölzl , monotone doesn't mean what you think it means
Johannes Hölzl (Mar 29 2018 at 08:20):
What is the difference between https://github.com/leanprover/mathlib/blob/master/order/basic.lean#L19
def monotone (f : α → β) := ∀⦃a b⦄, a ≤ b → f a ≤ f b
and
class is_ord_hom (f : α → α) : Prop := (ord : ∀ x y, x ≤ y → f x ≤ f y)
?
Monotone is a little bit more general, but not a type class...
Kenny Lau (Mar 29 2018 at 08:21):
@Johannes Hölzl monotone means increasing or decreasing
Kenny Lau (Mar 29 2018 at 08:21):
at least in where I'm from
Johannes Hölzl (Mar 29 2018 at 08:25):
Not in order theory, the "Monotonicity in order theory" section in https://en.wikipedia.org/wiki/Monotonic_function tells us that it means what you maybe call an increasing function.
Kenny Lau (Mar 29 2018 at 08:26):
fair enough
Last updated: Dec 20 2023 at 11:08 UTC