Monotone finite sequences #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove simp
lemmas that allow to simplify propositions like monotone ![a, b, c]
.
@[simp]
theorem
strict_mono_vec_cons
{α : Type u_1}
[preorder α]
{n : ℕ}
{f : fin (n + 1) → α}
{a : α} :
strict_mono (matrix.vec_cons a f) ↔ a < f 0 ∧ strict_mono f
@[simp]
theorem
strict_anti_vec_cons
{α : Type u_1}
[preorder α]
{n : ℕ}
{f : fin (n + 1) → α}
{a : α} :
strict_anti (matrix.vec_cons a f) ↔ f 0 < a ∧ strict_anti f
theorem
strict_mono.vec_cons
{α : Type u_1}
[preorder α]
{n : ℕ}
{f : fin (n + 1) → α}
{a : α}
(hf : strict_mono f)
(ha : a < f 0) :
strict_mono (matrix.vec_cons a f)
theorem
strict_anti.vec_cons
{α : Type u_1}
[preorder α]
{n : ℕ}
{f : fin (n + 1) → α}
{a : α}
(hf : strict_anti f)
(ha : f 0 < a) :
strict_anti (matrix.vec_cons a f)