This module provides typeclass instances and lemmas about order-related typeclasses.
Equations
- Std.instTransLeOfIsPreorder = { trans := ⋯ }
Equations
- Std.instTransLeOfIsPreorder_1 = { trans := ⋯ }
instance
Std.instIrreflLtOfIsPreorderOfLawfulOrderLT
{α : Type u}
[LT α]
[LE α]
[IsPreorder α]
[LawfulOrderLT α]
:
instance
Std.instTransLtOfLeOfLawfulOrderLT
{α : Type u}
[LT α]
[LE α]
[Trans (fun (x1 x2 : α) => x1 ≤ x2) (fun (x1 x2 : α) => x1 ≤ x2) fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderLT α]
:
Equations
- Std.instTransLtOfLeOfLawfulOrderLT = { trans := ⋯ }
instance
Std.instTransNotLtOfLawfulOrderLTOfTotalOfLe
{α : Type u}
{x✝ : LT α}
[LE α]
[LawfulOrderLT α]
[Total fun (x1 x2 : α) => x1 ≤ x2]
[Trans (fun (x1 x2 : α) => x1 ≤ x2) (fun (x1 x2 : α) => x1 ≤ x2) fun (x1 x2 : α) => x1 ≤ x2]
:
Equations
- Std.instTransNotLtOfLawfulOrderLTOfTotalOfLe = { trans := ⋯ }
theorem
Std.min_le_left
{α : Type u}
[Min α]
[LE α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderInf α]
{a b : α}
:
theorem
Std.min_le_right
{α : Type u}
[Min α]
[LE α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderInf α]
{a b : α}
:
instance
Std.instMinEqOrOfIsLinearOrderOfLawfulOrderInf
{α : Type u}
[LE α]
[Min α]
[IsLinearOrder α]
[LawfulOrderInf α]
:
MinEqOr α
theorem
Std.IsLinearOrder.of_refl_of_antisymm_of_lawfulOrderMin
{α : Type u}
[LE α]
[LE α]
[Min α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[Antisymm fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderMin α]
:
If a Min α
instance satisfies typical properties in terms of a reflexive and antisymmetric LE α
instance, then the LE α
instance represents a linear order.
instance
Std.instAssociativeMinOfIsLinearOrderOfLawfulOrderMin
{α : Type u}
[LE α]
[Min α]
[IsLinearOrder α]
[LawfulOrderMin α]
:
theorem
Std.left_le_max
{α : Type u}
[Max α]
[LE α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderSup α]
{a b : α}
:
theorem
Std.right_le_max
{α : Type u}
[Max α]
[LE α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderSup α]
{a b : α}
:
instance
Std.instMaxEqOrOfIsLinearOrderOfLawfulOrderSup
{α : Type u}
[LE α]
[Max α]
[IsLinearOrder α]
[LawfulOrderSup α]
:
MaxEqOr α
theorem
Std.IsLinearOrder.of_refl_of_antisymm_of_lawfulOrderMax
{α : Type u}
[LE α]
[Max α]
[Refl fun (x1 x2 : α) => x1 ≤ x2]
[Antisymm fun (x1 x2 : α) => x1 ≤ x2]
[LawfulOrderMax α]
:
If a Max α
instance satisfies typical properties in terms of a reflexive and antisymmetric LE α
instance, then the LE α
instance represents a linear order.
instance
Std.instAssociativeMaxOfIsLinearOrderOfLawfulOrderMax
{α : Type u}
[LE α]
[Max α]
[IsLinearOrder α]
[LawfulOrderMax α]
: