Type synonyms #
This file provides three type synonyms for order theory:
- OrderDual α: Type synonym of- αto equip it with the dual order (- a ≤ bbecomes- b ≤ a).
- Lex α: Type synonym of- αto equip it with its lexicographic order. The precise meaning depends on the type we take the lex of. Examples include- Prod,- Sigma,- List,- Finset.
- Colex α: Type synonym of- αto equip it with its colexicographic order. The precise meaning depends on the type we take the colex of. Examples include- Finset.
Notation #
αᵒᵈ is notation for OrderDual α.
The general rule for notation of Lex types is to append ₗ to the usual notation.
Implementation notes #
One should not abuse definitional equality between α and αᵒᵈ/Lex α. Instead, explicit
coercions should be inserted:
- OrderDual:- OrderDual.toDual : α → αᵒᵈand- OrderDual.ofDual : αᵒᵈ → α
- Lex:- toLex : α → Lex αand- ofLex : Lex α → α.
- Colex:- toColex : α → Colex αand- ofColex : Colex α → α.
See also #
This file is similar to Algebra.Group.TypeTags.
Order dual #
def
OrderDual.rec
{α : Type u_1}
{motive : αᵒᵈ → Sort u_2}
(toDual : (a : α) → motive (toDual a))
(a : αᵒᵈ)
 :
motive a
Recursor for αᵒᵈ.
Equations
- OrderDual.rec toDual = toDual
Instances For
Alias of the reverse direction of OrderDual.toDual_le_toDual.
Alias of the reverse direction of OrderDual.toDual_lt_toDual.
theorem
LE.le.ofDual
{α : Type u_1}
[LE α]
{a b : αᵒᵈ}
 :
b ≤ a → OrderDual.ofDual a ≤ OrderDual.ofDual b
Alias of the reverse direction of OrderDual.ofDual_le_ofDual.
theorem
LT.lt.ofDual
{α : Type u_1}
[LT α]
{a b : αᵒᵈ}
 :
b < a → OrderDual.ofDual a < OrderDual.ofDual b
Alias of the reverse direction of OrderDual.ofDual_lt_ofDual.