mathlib3 documentation

order.synonym

Type synonyms #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file provides two type synonyms for order theory:

Notation #

αᵒᵈ is notation for order_dual α.

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:

In fact, those are bundled as equivs to put goals in the right syntactic form for rewriting with the equiv API (⇑to_lex a where is coe_fn : (α ≃ lex α) → α → lex α, instead of a bare to_lex a).

See also #

This file is similar to algebra.group.type_tags.

Order dual #

@[protected, instance]
def order_dual.nontrivial {α : Type u_1} [h : nontrivial α] :
def order_dual.to_dual {α : Type u_1} :
α αᵒᵈ

to_dual is the identity function to the order_dual of a linear order.

Equations
def order_dual.of_dual {α : Type u_1} :
αᵒᵈ α

of_dual is the identity function from the order_dual of a linear order.

Equations
@[simp]
theorem order_dual.to_dual_inj {α : Type u_1} {a b : α} :
@[simp]
@[simp]
@[simp]
theorem order_dual.le_to_dual {α : Type u_1} [has_le α] {a : αᵒᵈ} {b : α} :
theorem order_dual.lt_to_dual {α : Type u_1} [has_lt α] {a : αᵒᵈ} {b : α} :
theorem order_dual.to_dual_le {α : Type u_1} [has_le α] {a : α} {b : αᵒᵈ} :
theorem order_dual.to_dual_lt {α : Type u_1} [has_lt α] {a : α} {b : αᵒᵈ} :
@[protected]
def order_dual.rec {α : Type u_1} {C : αᵒᵈ Sort u_2} (h₂ : Π (a : α), C (order_dual.to_dual a)) (a : αᵒᵈ) :
C a

Recursor for αᵒᵈ.

Equations
@[protected, simp]
theorem order_dual.forall {α : Type u_1} {p : αᵒᵈ Prop} :
( (a : αᵒᵈ), p a) (a : α), p (order_dual.to_dual a)
@[protected, simp]
theorem order_dual.exists {α : Type u_1} {p : αᵒᵈ Prop} :
( (a : αᵒᵈ), p a) (a : α), p (order_dual.to_dual a)
theorem has_le.le.dual {α : Type u_1} [has_le α] {a b : α} :

Alias of the reverse direction of order_dual.to_dual_le_to_dual.

theorem has_lt.lt.dual {α : Type u_1} [has_lt α] {a b : α} :

Alias of the reverse direction of order_dual.to_dual_lt_to_dual.

Alias of the reverse direction of order_dual.of_dual_le_of_dual.

theorem has_lt.lt.of_dual {α : Type u_1} [has_lt α] {a b : αᵒᵈ} :

Alias of the reverse direction of order_dual.of_dual_lt_of_dual.

Lexicographic order #

def lex (α : Type u_1) :
Type u_1

A type synonym to equip a type with its lexicographic order.

Equations
Instances for lex
def to_lex {α : Type u_1} :
α lex α

to_lex is the identity function to the lex of a type.

Equations
def of_lex {α : Type u_1} :
lex α α

of_lex is the identity function from the lex of a type.

Equations
@[simp]
theorem to_lex_symm_eq {α : Type u_1} :
@[simp]
theorem of_lex_symm_eq {α : Type u_1} :
@[simp]
theorem to_lex_of_lex {α : Type u_1} (a : lex α) :
@[simp]
theorem of_lex_to_lex {α : Type u_1} (a : α) :
@[simp]
theorem to_lex_inj {α : Type u_1} {a b : α} :
@[simp]
theorem of_lex_inj {α : Type u_1} {a b : lex α} :
@[protected]
def lex.rec {α : Type u_1} {β : lex α Sort u_2} (h : Π (a : α), β (to_lex a)) (a : lex α) :
β a

A recursor for lex. Use as induction x using lex.rec.

Equations