Skip to content

Commit 34dea34

Browse files
committed
feat: lemmas about WithBot.unbot (#6124)
1 parent 86c30b0 commit 34dea34

File tree

1 file changed

+9
-0
lines changed

1 file changed

+9
-0
lines changed

Mathlib/Order/WithBot.lean

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -249,6 +249,11 @@ theorem le_unbot_iff {a : α} {b : WithBot α} (h : b ≠ ⊥) :
249249
match b, h with
250250
| some _, _ => simp only [unbot_coe, coe_le_coe]
251251

252+
theorem unbot_le_iff {a : WithBot α} (h : a ≠ ⊥) {b : α} :
253+
unbot a h ≤ b ↔ a ≤ (b : WithBot α) := by
254+
match a, h with
255+
| some _, _ => simp only [unbot_coe, coe_le_coe]
256+
252257
end LE
253258

254259
section LT
@@ -870,6 +875,10 @@ theorem untop_le_iff {a : WithTop α} {b : α} (h : a ≠ ⊤) :
870875
untop a h ≤ b ↔ a ≤ (b : WithTop α) :=
871876
@WithBot.le_unbot_iff αᵒᵈ _ _ _ _
872877

878+
theorem le_untop_iff {a : α} {b : WithTop α} (h : b ≠ ⊤) :
879+
a ≤ untop b h ↔ (a : WithTop α) ≤ b :=
880+
@WithBot.unbot_le_iff αᵒᵈ _ _ _ _
881+
873882
end LE
874883

875884
section LT

0 commit comments

Comments
 (0)