File tree Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -249,6 +249,11 @@ theorem le_unbot_iff {a : α} {b : WithBot α} (h : b ≠ ⊥) :
249
249
match b, h with
250
250
| some _, _ => simp only [unbot_coe, coe_le_coe]
251
251
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
+
252
257
end LE
253
258
254
259
section LT
@@ -870,6 +875,10 @@ theorem untop_le_iff {a : WithTop α} {b : α} (h : a ≠ ⊤) :
870
875
untop a h ≤ b ↔ a ≤ (b : WithTop α) :=
871
876
@WithBot.le_unbot_iff αᵒᵈ _ _ _ _
872
877
878
+ theorem le_untop_iff {a : α} {b : WithTop α} (h : b ≠ ⊤) :
879
+ a ≤ untop b h ↔ (a : WithTop α) ≤ b :=
880
+ @WithBot.unbot_le_iff αᵒᵈ _ _ _ _
881
+
873
882
end LE
874
883
875
884
section LT
You can’t perform that action at this time.
0 commit comments