Documentation

Mathlib.Order.Category.PartOrd

Category of partial orders #

This defines PartOrd, the category of partial orders with monotone maps.

structure PartOrd :
Type (u_1 + 1)

The category of partial orders.

  • of :: (
    • carrier : Type u_1

      The underlying partially ordered type.

    • str : PartialOrder self
  • )
Instances For
    structure PartOrd.Hom (X Y : PartOrd) :

    The type of morphisms in PartOrd R.

    Instances For
      theorem PartOrd.Hom.ext_iff {X Y : PartOrd} {x y : X.Hom Y} :
      x = y x.hom' = y.hom'
      theorem PartOrd.Hom.ext {X Y : PartOrd} {x y : X.Hom Y} (hom' : x.hom' = y.hom') :
      x = y
      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.
      @[reducible, inline]
      abbrev PartOrd.Hom.hom {X Y : PartOrd} (f : X.Hom Y) :
      X →o Y

      Turn a morphism in PartOrd back into a OrderHom.

      Equations
      Instances For
        @[reducible, inline]
        abbrev PartOrd.ofHom {X Y : Type u} [PartialOrder X] [PartialOrder Y] (f : X →o Y) :
        { carrier := X, str := inst✝ } { carrier := Y, str := inst✝¹ }

        Typecheck a OrderHom as a morphism in PartOrd.

        Equations
        Instances For
          def PartOrd.Hom.Simps.hom (X Y : PartOrd) (f : X.Hom Y) :
          X →o Y

          Use the ConcreteCategory.hom projection for @[simps] lemmas.

          Equations
          Instances For

            The results below duplicate the ConcreteCategory simp lemmas, but we can keep them for dsimp.

            theorem PartOrd.ext {X Y : PartOrd} {f g : X Y} (w : ∀ (x : X), (CategoryTheory.ConcreteCategory.hom f) x = (CategoryTheory.ConcreteCategory.hom g) x) :
            f = g
            theorem PartOrd.coe_of (X : Type u) [PartialOrder X] :
            { carrier := X, str := inst✝ } = X
            @[simp]
            theorem PartOrd.hom_comp {X Y Z : PartOrd} (f : X Y) (g : Y Z) :
            theorem PartOrd.hom_ext {X Y : PartOrd} {f g : X Y} (hf : Hom.hom f = Hom.hom g) :
            f = g
            theorem PartOrd.hom_ext_iff {X Y : PartOrd} {f g : X Y} :
            @[simp]
            theorem PartOrd.hom_ofHom {X Y : Type u} [PartialOrder X] [PartialOrder Y] (f : X →o Y) :
            @[simp]
            theorem PartOrd.ofHom_hom {X Y : PartOrd} (f : X Y) :
            @[simp]
            theorem PartOrd.ofHom_id {X : Type u} [PartialOrder X] :
            ofHom OrderHom.id = CategoryTheory.CategoryStruct.id { carrier := X, str := inst✝ }
            @[simp]
            Equations
            • One or more equations did not get rendered due to their size.
            def PartOrd.Iso.mk {α β : PartOrd} (e : α ≃o β) :
            α β

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

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

              OrderDual as a functor.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[simp]
                theorem PartOrd.dual_map {X✝ Y✝ : PartOrd} (f : X✝ Y✝) :

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

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

                  Antisymmetrization as a functor. It is the free functor.

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

                    preordToPartOrd is left adjoint to the forgetful functor, meaning it is the free functor from Preord to PartOrd.

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

                      PreordToPartOrd and OrderDual commute.

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