The categories of semilattices #
This defines SemilatSupCat
and SemilatInfCat
, the categories of sup-semilattices with a bottom
element and inf-semilattices with a top element.
References #
The category of sup-semilattices with a bottom element.
- X : Type u
The underlying type of a sup-semilattice with a bottom element.
- isSemilatticeSup : SemilatticeSup self.X
- isOrderBot : OrderBot self.X
Instances For
The category of inf-semilattices with a top element.
- X : Type u
The underlying type of an inf-semilattice with a top element.
- isSemilatticeInf : SemilatticeInf self.X
- isOrderTop : OrderTop self.X
Instances For
Equations
- SemilatSupCat.instCoeSortType = { coe := SemilatSupCat.X }
@[simp]
Equations
- SemilatSupCat.instInhabited = { default := SemilatSupCat.of PUnit.{?u.3 + 1} }
Equations
- X.instFunLike Y = inferInstance
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.
@[simp]
theorem
SemilatSupCat.coe_forget_to_partOrd
(X : SemilatSupCat)
:
↑((CategoryTheory.forget₂ SemilatSupCat PartOrd).obj X) = X.X
Equations
- SemilatInfCat.instCoeSortType = { coe := SemilatInfCat.X }
@[simp]
Equations
- SemilatInfCat.instInhabited = { default := SemilatInfCat.of PUnit.{?u.3 + 1} }
Equations
- X.instFunLike Y = inferInstance
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.
@[simp]
theorem
SemilatInfCat.coe_forget_to_partOrd
(X : SemilatInfCat)
:
↑((CategoryTheory.forget₂ SemilatInfCat PartOrd).obj X) = X.X
Order dual #
Constructs an isomorphism of lattices from an order isomorphism between them.
Equations
- SemilatSupCat.Iso.mk e = { hom := { toFun := ⇑e, map_sup' := ⋯, map_bot' := ⋯ }, inv := { toFun := ⇑e.symm, map_sup' := ⋯, map_bot' := ⋯ }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
@[simp]
OrderDual
as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
Constructs an isomorphism of lattices from an order isomorphism between them.
Equations
- SemilatInfCat.Iso.mk e = { hom := { toFun := ⇑e, map_inf' := ⋯, map_top' := ⋯ }, inv := { toFun := ⇑e.symm, map_inf' := ⋯, map_top' := ⋯ }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
@[simp]
OrderDual
as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
The equivalence between SemilatSupCat
and SemilatInfCat
induced by OrderDual
both ways.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]