Documentation

Mathlib.Deprecated.Sort

The predicate List.Sorted (now deprecated). #

@[deprecated List.Pairwise (since := "2025-10-11")]
def List.Sorted {α : Type u} (R : ααProp) :
List αProp

Sorted r l is the same as List.Pairwise r l and has been deprecated. Consider using any of SortedLE, SortedLT, SortedGE, or SortedGT if the relation you're using is a preorder.

Equations
Instances For
    @[deprecated List.instDecidablePairwise (since := "2025-10-11")]
    def List.decidableSorted {α : Type u} {r : ααProp} [DecidableRel r] (l : List α) :

    Deprecated decidable instance for Sorted.

    Equations
    Instances For
      @[deprecated List.Pairwise.nil (since := "2025-10-11")]
      theorem List.sorted_nil {α : Type u} {r : ααProp} :
      @[deprecated List.Pairwise.of_cons (since := "2025-10-11")]
      theorem List.Sorted.of_cons {α : Type u} {r : ααProp} {a : α} {l : List α} (p : Sorted r (a :: l)) :
      Sorted r l
      @[deprecated List.Pairwise.tail (since := "2025-10-11")]
      theorem List.Sorted.tail {α : Type u} {r : ααProp} {l : List α} (h : Sorted r l) :
      @[deprecated List.rel_of_pairwise_cons (since := "2025-10-11")]
      theorem List.rel_of_sorted_cons {α : Type u} {r : ααProp} {a : α} {l : List α} (p : Sorted r (a :: l)) {a' : α} :
      a' lr a a'
      @[deprecated List.pairwise_cons (since := "2025-10-11")]
      theorem List.sorted_cons {α : Type u} {r : ααProp} {a : α} {l : List α} :
      Sorted r (a :: l) (∀ (a' : α), a' lr a a') Sorted r l
      @[deprecated List.Pairwise.filter (since := "2025-10-11")]
      theorem List.Sorted.filter {α : Type u} {r : ααProp} {l : List α} (p : αBool) :
      Sorted r lSorted r (List.filter p l)
      @[deprecated List.pairwise_singleton (since := "2025-10-11")]
      theorem List.sorted_singleton {α : Type u} (r : ααProp) (a : α) :
      @[deprecated List.Pairwise.rel_of_mem_take_of_mem_drop (since := "2025-10-11")]
      theorem List.Sorted.rel_of_mem_take_of_mem_drop {α : Type u} {r : ααProp} {l : List α} {x y : α} {i : Nat} (h : Sorted r l) (hx : x take i l) (hy : y drop i l) :
      r x y
      @[deprecated List.Pairwise.filterMap (since := "2025-10-11")]
      theorem List.Sorted.filterMap {α : Type u} {r : ααProp} {l : List α} (f : αOption α) {s : ααProp} (H : ∀ (a a' : α), r a a'∀ (b : α), f a = some b∀ (b' : α), f a' = some b's b b') :
      Sorted r lSorted s (List.filterMap f l)