Documentation

Mathlib.Order.Category.PartOrdEmb

Category of partial orders, with order embeddings as morphisms #

This defines PartOrdEmb, the category of partial orders with order embeddings as morphisms. We also show that PartOrdEmb has filtered colimits.

structure PartOrdEmb :
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 PartOrdEmb.Hom (X Y : PartOrdEmb) :

    The type of morphisms in PartOrdEmb R.

    Instances For
      theorem PartOrdEmb.Hom.ext {X Y : PartOrdEmb} {x y : X.Hom Y} (hom' : x.hom' = y.hom') :
      x = y
      theorem PartOrdEmb.Hom.ext_iff {X Y : PartOrdEmb} {x y : X.Hom Y} :
      x = y x.hom' = y.hom'
      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 PartOrdEmb.Hom.hom {X Y : PartOrdEmb} (f : X.Hom Y) :
      X ↪o Y

      Turn a morphism in PartOrdEmb back into a OrderEmbedding.

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

        Typecheck a OrderEmbedding as a morphism in PartOrdEmb.

        Equations
        Instances For
          def PartOrdEmb.Hom.Simps.hom (X Y : PartOrdEmb) (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 PartOrdEmb.ext {X Y : PartOrdEmb} {f g : X Y} (w : ∀ (x : X), (CategoryTheory.ConcreteCategory.hom f) x = (CategoryTheory.ConcreteCategory.hom g) x) :
            f = g
            theorem PartOrdEmb.coe_of (X : Type u) [PartialOrder X] :
            { carrier := X, str := inst✝ } = X
            theorem PartOrdEmb.hom_ext {X Y : PartOrdEmb} {f g : X Y} (hf : Hom.hom f = Hom.hom g) :
            f = g
            theorem PartOrdEmb.hom_ext_iff {X Y : PartOrdEmb} {f g : X Y} :
            @[simp]
            theorem PartOrdEmb.hom_ofHom {X Y : Type u} [PartialOrder X] [PartialOrder Y] (f : X ↪o Y) :
            @[simp]
            theorem PartOrdEmb.ofHom_hom {X Y : PartOrdEmb} (f : X Y) :
            @[simp]
            theorem PartOrdEmb.ofHom_id {X : Type u} [PartialOrder X] :
            ofHom (RelEmbedding.refl fun (x1 x2 : X) => x1 x2) = CategoryTheory.CategoryStruct.id { carrier := X, str := inst✝ }
            Equations
            • One or more equations did not get rendered due to their size.
            def PartOrdEmb.Iso.mk {α β : PartOrdEmb} (e : α ≃o β) :
            α β

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

            Equations
            Instances For
              @[simp]
              theorem PartOrdEmb.Iso.mk_inv {α β : PartOrdEmb} (e : α ≃o β) :
              @[simp]
              theorem PartOrdEmb.Iso.mk_hom {α β : PartOrdEmb} (e : α ≃o β) :

              OrderDual as a functor.

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

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

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

                  Given a functor F : J ⥤ PartOrdEmb and a colimit cocone c for F ⋙ forget _, this is the type c.pt on which we define a partial order which makes it the colimit of F.

                  Equations
                  Instances For

                    The colimit cocone for a functor F : J ⥤ PartOrdEmb from a filtered category that is constructed from a colimit cocone for F ⋙ forget _.

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

                      A colimit cocone for F : J ⥤ PartOrdEmb (with J filtered) can be obtained from a colimit cocone for F ⋙ forget _.

                      Equations
                      Instances For