Zulip Chat Archive
Stream: Is there code for X?
Topic: If `f x ≤ f y → x ≤ y`, then `f` is injective
Anne Baanen (Jul 19 2021 at 13:15):
I can't quite find the following result in the library:
lemma injective_of_le_imp_le {α β : Type*} [partial_order α] [preorder β] (f : α → β)
(h : ∀ {x y}, f x ≤ f y → x ≤ y) : function.injective f :=
λ x y hxy, le_antisymm (h hxy.le) (h hxy.ge)
(In fact, I have docs#strict_mono since f x ≤ f y ↔ x ≤ y
, but docs#strict_mono.injective requires a linear_order
assumption.)
Anne Baanen (Jul 19 2021 at 13:15):
The closest I could find was docs#injective_of_lt_imp_ne, but that again requires linear_order
.
Anne Baanen (Jul 20 2021 at 13:27):
Since there isn't any response: #8373
Last updated: Dec 20 2023 at 11:08 UTC