@@ -207,15 +207,6 @@ lemma not_coe_le_bot (a : α) : ¬(a : WithBot α) ≤ ⊥ := by simp [le_def]
207
207
208
208
instance orderBot : OrderBot (WithBot α) where bot_le := by simp [le_def]
209
209
210
- -- TODO: This deprecated lemma is still used (through simp)
211
- @[simp, deprecated coe_le_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
212
- theorem some_le_some : @LE.le (WithBot α) _ (Option.some a) (Option.some b) ↔ a ≤ b :=
213
- coe_le_coe
214
-
215
- -- TODO: This deprecated lemma is still used (through simp)
216
- @[simp, deprecated bot_le "Don't mix Option and WithBot" (since := "2024-05-27")]
217
- theorem none_le {a : WithBot α} : @LE.le (WithBot α) _ none a := bot_le
218
-
219
210
instance orderTop [OrderTop α] : OrderTop (WithBot α) where le_top x := by cases x <;> simp [le_def]
220
211
221
212
instance instBoundedOrder [OrderTop α] : BoundedOrder (WithBot α) :=
@@ -258,18 +249,6 @@ lemma lt_def : x < y ↔ ∃ b : α, y = ↑b ∧ ∀ a : α, x = ↑a → a < b
258
249
@[simp] lemma bot_lt_coe (a : α) : ⊥ < (a : WithBot α) := by simp [lt_def]
259
250
@[simp] protected lemma not_lt_bot (a : WithBot α) : ¬a < ⊥ := by simp [lt_def]
260
251
261
- -- TODO: This deprecated lemma is still used (through simp)
262
- @[simp, deprecated coe_lt_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
263
- theorem some_lt_some : @LT.lt (WithBot α) _ (Option.some a) (Option.some b) ↔ a < b := coe_lt_coe
264
-
265
- -- TODO: This deprecated lemma is still used (through simp)
266
- @[simp, deprecated bot_lt_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
267
- theorem none_lt_some (a : α) : @LT.lt (WithBot α) _ none (some a) := bot_lt_coe _
268
-
269
- -- TODO: This deprecated lemma is still used (through simp)
270
- @[simp, deprecated not_lt_bot "Don't mix Option and WithBot" (since := "2024-05-27")]
271
- theorem not_lt_none (a : WithBot α) : ¬@LT.lt (WithBot α) _ a none := WithBot.not_lt_bot _
272
-
273
252
lemma lt_iff_exists_coe : x < y ↔ ∃ b : α, y = b ∧ x < b := by cases y <;> simp
274
253
275
254
lemma lt_coe_iff : x < b ↔ ∀ a : α, x = a → a < b := by simp [lt_def]
@@ -709,17 +688,8 @@ lemma le_def : x ≤ y ↔ ∀ b : α, y = ↑b → ∃ a : α, x = ↑a ∧ a
709
688
710
689
lemma not_top_le_coe (a : α) : ¬ ⊤ ≤ (a : WithTop α) := by simp [le_def]
711
690
712
- -- TODO: This deprecated lemma is still used (through simp)
713
- @[simp, deprecated coe_le_coe "Don't mix Option and WithTop" (since := "2024-05-27")]
714
- theorem some_le_some : @LE.le (WithTop α) _ (Option.some a) (Option.some b) ↔ a ≤ b :=
715
- coe_le_coe
716
-
717
691
instance orderTop : OrderTop (WithTop α) where le_top := by simp [le_def]
718
692
719
- -- TODO: This deprecated lemma is still used (through simp)
720
- @[simp, deprecated le_top "Don't mix Option and WithTop" (since := "2024-05-27")]
721
- theorem le_none {a : WithTop α} : @LE.le (WithTop α) _ a none := le_top
722
-
723
693
instance orderBot [OrderBot α] : OrderBot (WithTop α) where bot_le x := by cases x <;> simp [le_def]
724
694
725
695
instance boundedOrder [OrderBot α] : BoundedOrder (WithTop α) :=
@@ -762,15 +732,6 @@ lemma lt_def : x < y ↔ ∃ a : α, x = ↑a ∧ ∀ b : α, y = ↑b → a < b
762
732
@[simp] lemma coe_lt_top (a : α) : (a : WithTop α) < ⊤ := by simp [lt_def]
763
733
@[simp] protected lemma not_top_lt (a : WithTop α) : ¬⊤ < a := by simp [lt_def]
764
734
765
- @[simp, deprecated coe_lt_coe "Don't mix Option and WithTop" (since := "2024-05-27")]
766
- theorem some_lt_some : @LT.lt (WithTop α) _ (Option.some a) (Option.some b) ↔ a < b := coe_lt_coe
767
-
768
- @[simp, deprecated coe_lt_top "Don't mix Option and WithTop" (since := "2024-05-27")]
769
- theorem some_lt_none (a : α) : @LT.lt (WithTop α) _ (Option.some a) none := coe_lt_top a
770
-
771
- @[simp, deprecated not_top_lt "Don't mix Option and WithTop" (since := "2024-05-27")]
772
- theorem not_none_lt (a : WithTop α) : ¬@LT.lt (WithTop α) _ none a := WithTop.not_top_lt _
773
-
774
735
lemma lt_iff_exists_coe : x < y ↔ ∃ a : α, x = a ∧ a < y := by cases x <;> simp
775
736
776
737
lemma coe_lt_iff : a < y ↔ ∀ b : α, y = b → a < b := by simp [lt_def]
0 commit comments