Skip to content

Commit fcc2138

Browse files
committed
chore(Order): deprecate Codisjoint.ne_bot_of_ne_top', OrderEmbedding.{w,}covBy_of_apply and OrderIso.map_{w,}covBy (#28486)
1 parent ec382b5 commit fcc2138

File tree

3 files changed

+10
-27
lines changed

3 files changed

+10
-27
lines changed

Mathlib/Order/Cover.lean

Lines changed: 6 additions & 24 deletions
Original file line numberDiff line numberDiff line change
@@ -120,18 +120,9 @@ alias ⟨_, WCovBy.toDual⟩ := toDual_wcovBy_toDual_iff
120120

121121
alias ⟨_, WCovBy.ofDual⟩ := ofDual_wcovBy_ofDual_iff
122122

123-
theorem OrderEmbedding.wcovBy_of_apply {α β : Type*} [Preorder α] [Preorder β]
124-
(f : α ↪o β) {x y : α} (h : f x ⩿ f y) : x ⩿ y := by
125-
use f.le_iff_le.1 h.1
126-
intro a
127-
rw [← f.lt_iff_lt, ← f.lt_iff_lt]
128-
apply h.2
129-
130-
theorem OrderIso.map_wcovBy {α β : Type*} [Preorder α] [Preorder β]
131-
(f : α ≃o β) {x y : α} : f x ⩿ f y ↔ x ⩿ y := by
132-
use f.toOrderEmbedding.wcovBy_of_apply
133-
conv_lhs => rw [← f.symm_apply_apply x, ← f.symm_apply_apply y]
134-
exact f.symm.toOrderEmbedding.wcovBy_of_apply
123+
@[deprecated (since := "2025-11-07")] alias OrderEmbedding.wcovBy_of_apply := WCovBy.of_image
124+
125+
@[deprecated (since := "2025-11-07")] alias OrderIso.map_wcovBy := apply_wcovBy_apply_iff
135126

136127
end Preorder
137128

@@ -309,18 +300,9 @@ theorem apply_covBy_apply_iff {E : Type*} [EquivLike E α β] [OrderIsoClass E
309300
theorem covBy_of_eq_or_eq (hab : a < b) (h : ∀ c, a ≤ c → c ≤ b → c = a ∨ c = b) : a ⋖ b :=
310301
⟨hab, fun c ha hb => (h c ha.le hb.le).elim ha.ne' hb.ne⟩
311302

312-
theorem OrderEmbedding.covBy_of_apply {α β : Type*} [Preorder α] [Preorder β]
313-
(f : α ↪o β) {x y : α} (h : f x ⋖ f y) : x ⋖ y := by
314-
use f.lt_iff_lt.1 h.1
315-
intro a
316-
rw [← f.lt_iff_lt, ← f.lt_iff_lt]
317-
apply h.2
318-
319-
theorem OrderIso.map_covBy {α β : Type*} [Preorder α] [Preorder β]
320-
(f : α ≃o β) {x y : α} : f x ⋖ f y ↔ x ⋖ y := by
321-
use f.toOrderEmbedding.covBy_of_apply
322-
conv_lhs => rw [← f.symm_apply_apply x, ← f.symm_apply_apply y]
323-
exact f.symm.toOrderEmbedding.covBy_of_apply
303+
@[deprecated (since := "2025-11-07")] alias OrderEmbedding.covBy_of_apply := CovBy.of_image
304+
305+
@[deprecated (since := "2025-11-07")] alias OrderIso.map_covBy := apply_covBy_apply_iff
324306

325307
end Preorder
326308

Mathlib/Order/Disjoint.lean

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -268,8 +268,9 @@ theorem bot_codisjoint : Codisjoint ⊥ a ↔ a = ⊤ :=
268268
lemma Codisjoint.ne_bot_of_ne_top (h : Codisjoint a b) (ha : a ≠ ⊤) : b ≠ ⊥ := by
269269
rintro rfl; exact ha <| by simpa using h
270270

271-
lemma Codisjoint.ne_bot_of_ne_top' (h : Codisjoint a b) (hb : b ≠ ⊤) : a ≠ ⊥ := by
272-
rintro rfl; exact hb <| by simpa using h
271+
@[deprecated ne_bot_of_ne_top (since := "2025-11-07")]
272+
lemma Codisjoint.ne_bot_of_ne_top' (h : Codisjoint a b) (hb : b ≠ ⊤) : a ≠ ⊥ :=
273+
ne_bot_of_ne_top h.symm hb
273274

274275
end PartialBoundedOrder
275276

Mathlib/Order/SuccPred/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -346,7 +346,7 @@ theorem _root_.OrderIso.map_succ [PartialOrder β] [SuccOrder β] (f : α ≃o
346346
f (succ a) = succ (f a) := by
347347
by_cases h : IsMax a
348348
· rw [h.succ_eq, (f.isMax_apply.2 h).succ_eq]
349-
· exact (f.map_covBy.2 <| covBy_succ_of_not_isMax h).succ_eq.symm
349+
· exact ((apply_covBy_apply_iff f).2 <| covBy_succ_of_not_isMax h).succ_eq.symm
350350

351351
section NoMaxOrder
352352

0 commit comments

Comments
 (0)