Documentation

Mathlib.Order.Category.BddOrd

The category of bounded orders #

This defines BddOrd, the category of bounded orders.

structure BddOrd :
Type (u_1 + 1)

The category of bounded orders with monotone functions.

Instances For
    def BddOrd.of (α : Type u_1) [PartialOrder α] [BoundedOrder α] :

    Construct a bundled BddOrd from a Fintype PartialOrder.

    Equations
    Instances For
      @[simp]
      theorem BddOrd.coe_of (α : Type u_1) [PartialOrder α] [BoundedOrder α] :
      (of α).toPartOrd = α
      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.
      Equations
      • One or more equations did not get rendered due to their size.

      OrderDual as a functor.

      Equations
      Instances For
        @[simp]
        @[simp]
        theorem BddOrd.dual_map {x✝ x✝¹ : BddOrd} (a : BoundedOrderHom x✝.toPartOrd x✝¹.toPartOrd) :
        def BddOrd.Iso.mk {α β : BddOrd} (e : α.toPartOrd ≃o β.toPartOrd) :
        α β

        Constructs an equivalence between bounded orders from an order isomorphism between them.

        Equations
        Instances For
          @[simp]
          theorem BddOrd.Iso.mk_inv {α β : BddOrd} (e : α.toPartOrd ≃o β.toPartOrd) :
          (mk e).inv = e.symm
          @[simp]
          theorem BddOrd.Iso.mk_hom {α β : BddOrd} (e : α.toPartOrd ≃o β.toPartOrd) :
          (mk e).hom = e

          The equivalence between BddOrd and itself induced by OrderDual both ways.

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