Documentation

Mathlib.Data.Fin.Tuple.Monotone

Monotone finite sequences #

In this file we prove simp lemmas that allow to simplify propositions like Monotone ![a, b, c].

theorem liftFun_vecCons {α : Type u_1} {n : } (r : ααProp) [IsTrans α r] {f : Fin (n + 1)α} {a : α} :
((fun (x x_1 : Fin (Nat.succ (n + 1))) => x < x_1) r) (Matrix.vecCons a f) (Matrix.vecCons a f) r a (f 0) ((fun (x x_1 : Fin (n + 1)) => x < x_1) r) f f
@[simp]
theorem strictMono_vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} :
@[simp]
theorem monotone_vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} :
@[simp]
theorem monotone_vecEmpty {α : Type u_1} [Preorder α] {a : α} :
@[simp]
theorem strictMono_vecEmpty {α : Type u_1} [Preorder α] {a : α} :
@[simp]
theorem strictAnti_vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} :
@[simp]
theorem antitone_vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} :
@[simp]
theorem antitone_vecEmpty {α : Type u_1} [Preorder α] {a : α} :
@[simp]
theorem strictAnti_vecEmpty {α : Type u_1} [Preorder α] {a : α} :
theorem StrictMono.vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} (hf : StrictMono f) (ha : a < f 0) :
theorem StrictAnti.vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} (hf : StrictAnti f) (ha : f 0 < a) :
theorem Monotone.vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} (hf : Monotone f) (ha : a f 0) :
theorem Antitone.vecCons {α : Type u_1} [Preorder α] {n : } {f : Fin (n + 1)α} {a : α} (hf : Antitone f) (ha : f 0 a) :