Orders #
Defines classes for preorders and partial orders and proves some basic lemmas about them.
A preorder is a reflexive, transitive relation ≤
with a < b
defined in the obvious way.
- le_refl : ∀ (a : α), a ≤ a
Instances
Alias of not_le_of_lt
.
Alias of not_lt_of_le
.
def
decidableLTOfDecidableLE
{α : Type u_1}
[Preorder α]
[DecidableRel fun (x1 x2 : α) => x1 ≤ x2]
:
DecidableRel fun (x1 x2 : α) => x1 < x2
<
is decidable if ≤
is.
Equations
Instances For
Definition of PartialOrder
and lemmas about types with a partial order #
A partial order is a reflexive, transitive, antisymmetric relation ≤
.
Instances
Alias of le_antisymm
.
def
decidableEqOfDecidableLE
{α : Type u_1}
[PartialOrder α]
[DecidableRel fun (x1 x2 : α) => x1 ≤ x2]
:
Equality is decidable if ≤
is.
Equations
Instances For
theorem
Decidable.lt_or_eq_of_le
{α : Type u_1}
[PartialOrder α]
{a b : α}
[DecidableRel fun (x1 x2 : α) => x1 ≤ x2]
(hab : a ≤ b)
:
theorem
Decidable.eq_or_lt_of_le
{α : Type u_1}
[PartialOrder α]
{a b : α}
[DecidableRel fun (x1 x2 : α) => x1 ≤ x2]
(hab : a ≤ b)
:
theorem
Decidable.le_iff_lt_or_eq
{α : Type u_1}
[PartialOrder α]
{a b : α}
[DecidableRel fun (x1 x2 : α) => x1 ≤ x2]
: