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

Commit 11e3047

Browse files
committed
feat(algebra/ordered_monoid): min_top_(left|right) (#8880)
1 parent e290569 commit 11e3047

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

src/algebra/ordered_monoid.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -140,6 +140,10 @@ lemma top_add (a : α) : ⊤ + a = ⊤ := linear_ordered_add_comm_monoid_with_to
140140
lemma add_top (a : α) : a + ⊤ = ⊤ :=
141141
trans (add_comm _ _) (top_add _)
142142

143+
-- TODO: Generalize to a not-yet-existing typeclass extending `linear_order` and `order_top`
144+
@[simp] lemma min_top_left (a : α) : min (⊤ : α) a = a := min_eq_right le_top
145+
@[simp] lemma min_top_right (a : α) : min a ⊤ = a := min_eq_left le_top
146+
143147
end linear_ordered_add_comm_monoid_with_top
144148

145149
/-- Pullback an `ordered_comm_monoid` under an injective map.

0 commit comments

Comments
 (0)