Documentation

Mathlib.Order.Category.OmegaCompletePartialOrder

Category of types with an omega complete partial order #

In this file, we bundle the class OmegaCompletePartialOrder into a concrete category and prove that continuous functions also form an OmegaCompletePartialOrder.

Main definitions #

structure ωCPO :
Type (u + 1)

The category of types with an omega complete partial order.

Instances For
    theorem ωCPO.coe_of (α : Type u_1) [OmegaCompletePartialOrder α] :
    { carrier := α, str := inst✝ }.carrier = α
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • One or more equations did not get rendered due to their size.

    The pi-type gives a cone for a product.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      The pi-type is a limit cone for the product.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def ωCPO.HasEqualizers.equalizerι {α : Type u_1} {β : Type u_2} [OmegaCompletePartialOrder α] [OmegaCompletePartialOrder β] (f g : α →𝒄 β) :
        { a : α // f a = g a } →𝒄 α

        The equalizer inclusion function as a ContinuousHom.

        Equations
        Instances For

          A construction of the equalizer fork.

          Equations
          Instances For

            The equalizer fork is a limit.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For