Documentation

Mathlib.Data.PSigma.Order

Lexicographic order on a sigma type #

This file defines the lexicographic order on Σₗ' i, α i. a is less than b if its summand is strictly less than the summand of b or they are in the same summand and a is less than b there.

Notation #

See also #

Related files are:

TODO #

Define the disjoint order on Σ' i, α i, where x ≤ y≤ y only if x.fst = y.fst. Prove that a sigma type is a NoMaxOrder, NoMinOrder, DenselyOrdered when its summands are.

The notation Σₗ' i, α i refers to a sigma type which is locall equipped with the lexicographic order.

Equations
  • One or more equations did not get rendered due to their size.
instance PSigma.Lex.le {ι : Type u_1} {α : ιType u_2} [inst : LT ι] [inst : (i : ι) → LE (α i)] :
LE (Lex ((i : ι) ×' α i))

The lexicographical ≤≤ on a sigma type.

Equations
  • PSigma.Lex.le = { le := PSigma.Lex (fun x x_1 => x < x_1) fun x x_1 x_2 => x_1 x_2 }
instance PSigma.Lex.lt {ι : Type u_1} {α : ιType u_2} [inst : LT ι] [inst : (i : ι) → LT (α i)] :
LT (Lex ((i : ι) ×' α i))

The lexicographical < on a sigma type.

Equations
  • PSigma.Lex.lt = { lt := PSigma.Lex (fun x x_1 => x < x_1) fun x x_1 x_2 => x_1 < x_2 }
instance PSigma.Lex.preorder {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] :
Preorder (Lex ((i : ι) ×' α i))
Equations
  • PSigma.Lex.preorder = let src := PSigma.Lex.le; let src_1 := PSigma.Lex.lt; Preorder.mk (_ : ∀ (x : Lex ((i : ι) ×' α i)), x x) (_ : ∀ (a b c : Lex ((i : ι) ×' α i)), a bb ca c)
instance PSigma.Lex.partialOrder {ι : Type u_1} {α : ιType u_2} [inst : PartialOrder ι] [inst : (i : ι) → PartialOrder (α i)] :
PartialOrder (Lex ((i : ι) ×' α i))

Dictionary / lexicographic partial_order for dependent pairs.

Equations
  • PSigma.Lex.partialOrder = let src := PSigma.Lex.preorder; PartialOrder.mk (_ : ∀ (a b : Lex ((i : ι) ×' α i)), a bb aa = b)
instance PSigma.Lex.linearOrder {ι : Type u_1} {α : ιType u_2} [inst : LinearOrder ι] [inst : (i : ι) → LinearOrder (α i)] :
LinearOrder (Lex ((i : ι) ×' α i))

Dictionary / lexicographic linear_order for pairs.

Equations
  • One or more equations did not get rendered due to their size.
instance PSigma.Lex.orderBot {ι : Type u_1} {α : ιType u_2} [inst : PartialOrder ι] [inst : OrderBot ι] [inst : (i : ι) → Preorder (α i)] [inst : OrderBot (α )] :
OrderBot (Lex ((i : ι) ×' α i))

The lexicographical linear order on a sigma type.

Equations
instance PSigma.Lex.orderTop {ι : Type u_1} {α : ιType u_2} [inst : PartialOrder ι] [inst : OrderTop ι] [inst : (i : ι) → Preorder (α i)] [inst : OrderTop (α )] :
OrderTop (Lex ((i : ι) ×' α i))

The lexicographical linear order on a sigma type.

Equations
instance PSigma.Lex.boundedOrder {ι : Type u_1} {α : ιType u_2} [inst : PartialOrder ι] [inst : BoundedOrder ι] [inst : (i : ι) → Preorder (α i)] [inst : OrderBot (α )] [inst : OrderTop (α )] :
BoundedOrder (Lex ((i : ι) ×' α i))

The lexicographical linear order on a sigma type.

Equations
  • PSigma.Lex.boundedOrder = let src := PSigma.Lex.orderBot; let src_1 := PSigma.Lex.orderTop; BoundedOrder.mk
instance PSigma.Lex.denselyOrdered {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : DenselyOrdered ι] [inst : ∀ (i : ι), Nonempty (α i)] [inst : (i : ι) → Preorder (α i)] [inst : ∀ (i : ι), DenselyOrdered (α i)] :
DenselyOrdered (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.denselyOrdered_of_noMaxOrder {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : ∀ (i : ι), DenselyOrdered (α i)] [inst : ∀ (i : ι), NoMaxOrder (α i)] :
DenselyOrdered (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.densely_ordered_of_noMinOrder {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : ∀ (i : ι), DenselyOrdered (α i)] [inst : ∀ (i : ι), NoMinOrder (α i)] :
DenselyOrdered (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.noMaxOrder_of_nonempty {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : NoMaxOrder ι] [inst : ∀ (i : ι), Nonempty (α i)] :
NoMaxOrder (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.noMinOrder_of_nonempty {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : NoMinOrder ι] [inst : ∀ (i : ι), Nonempty (α i)] :
NoMinOrder (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.noMaxOrder {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : ∀ (i : ι), NoMaxOrder (α i)] :
NoMaxOrder (Lex ((i : ι) ×' α i))
Equations
instance PSigma.Lex.noMinOrder {ι : Type u_1} {α : ιType u_2} [inst : Preorder ι] [inst : (i : ι) → Preorder (α i)] [inst : ∀ (i : ι), NoMinOrder (α i)] :
NoMinOrder (Lex ((i : ι) ×' α i))
Equations