Zulip Chat Archive
Stream: Is there code for X?
Topic: lt on functions
Eric Wieser (Feb 03 2021 at 14:14):
Does this exist somewhere?
lemma pi.lt_of_le_of_lt {α : Type*} {β : Type*} [preorder β]
{f g : α → β} (h : f ≤ g) {x : α} (hx : f x < g x) : f < g :=
begin
apply lt_of_le_not_le (pi.le_def.mpr h),
rw [pi.le_def, not_forall],
refine ⟨x, hx.not_le⟩,
end
Eric Wieser (Feb 03 2021 at 14:37):
Done in #6023
Last updated: Dec 20 2023 at 11:08 UTC