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.
The category of partial orders.
- of :: (
- carrier : Type u_1
The underlying partially ordered type.
- str : PartialOrder ↑self
- )
Instances For
Equations
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.
Turn a morphism in PartOrdEmb back into a OrderEmbedding.
Equations
Instances For
Typecheck a OrderEmbedding as a morphism in PartOrdEmb.
Equations
Instances For
Use the ConcreteCategory.hom projection for @[simps] lemmas.
Equations
- PartOrdEmb.Hom.Simps.hom X Y f = f.hom
Instances For
The results below duplicate the ConcreteCategory simp lemmas, but we can keep them for dsimp.
Equations
- One or more equations did not get rendered due to their size.
Constructs an equivalence between partial orders from an order isomorphism between them.
Equations
- PartOrdEmb.Iso.mk e = { hom := PartOrdEmb.ofHom (RelIso.toRelEmbedding e), inv := PartOrdEmb.ofHom (RelIso.toRelEmbedding e.symm), hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
OrderDual as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
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
Equations
- One or more equations did not get rendered due to their size.
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
Auxiliary definition for isColimitCocone.
Equations
- PartOrdEmb.Limits.CoconePt.desc hc s = { toFun := hc.desc ((CategoryTheory.forget PartOrdEmb).mapCocone s), inj' := ⋯, map_rel_iff' := ⋯ }
Instances For
A colimit cocone for F : J ⥤ PartOrdEmb (with J filtered) can be
obtained from a colimit cocone for F ⋙ forget _.
Equations
- PartOrdEmb.Limits.isColimitCocone hc = { desc := fun (s : CategoryTheory.Limits.Cocone F) => PartOrdEmb.ofHom (PartOrdEmb.Limits.CoconePt.desc hc s), fac := ⋯, uniq := ⋯ }