Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 3592f45

Browse files
committed
chore(order/filter/filter_product): fix const_lt, make const_lt_iff @[simp, norm_cast] (#17442)
1 parent 70a4f21 commit 3592f45

File tree

1 file changed

+2
-1
lines changed

1 file changed

+2
-1
lines changed

src/order/filter/filter_product.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -47,8 +47,9 @@ by simp only [lt_iff_le_not_le, eventually_and, coe_le, eventually_not, eventual
4747

4848
lemma coe_pos [preorder β] [has_zero β] {f : α → β} : 0 < (f : β*) ↔ ∀* x, 0 < f x := coe_lt
4949

50-
lemma const_lt [preorder β] {x y : β} : x y → (↑x : β*) ↑y := lift_rel_const
50+
lemma const_lt [preorder β] {x y : β} : x < y → (↑x : β*) < ↑y := coe_lt.mpr ∘ lift_rel_const
5151

52+
@[simp, norm_cast]
5253
lemma const_lt_iff [preorder β] {x y : β} : (↑x : β*) < ↑y ↔ x < y :=
5354
coe_lt.trans lift_rel_const_iff
5455

0 commit comments

Comments
 (0)