Documentation

Mathlib.Order.Extension.Linear

Extend a partial order to a linear order #

This file constructs a linear order which is an extension of the given partial order, using Zorn's lemma.

theorem extend_partialOrder {α : Type u} (r : ααProp) [IsPartialOrder α r] :
∃ (s : ααProp), IsLinearOrder α s r s

Any partial order can be extended to a linear order.

def LinearExtension (α : Type u) :

A type alias for α, intended to extend a partial order on α to a linear order.

Equations
Instances For
    Equations

    The embedding of α into LinearExtension α as an order homomorphism.

    Equations
    • toLinearExtension = { toFun := fun (x : α) => x, monotone' := }
    Instances For
      Equations
      • instInhabitedLinearExtension = { default := default }