The category of lattices #
This defines Lat
, the category of lattices.
Note that Lat
doesn't correspond to the literature definition of [Lat
]
(https://ncatlab.org/nlab/show/Lat) as we don't require bottom or top elements. Instead, Lat
corresponds to BddLat
.
TODO #
The free functor from Lat
to BddLat
is X → WithTop (WithBot X)
.
Equations
- Lat.instCoeSortType = CategoryTheory.Bundled.coeSort
Equations
- Lat.instInhabited = { default := Lat.of Bool }
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.
Constructs an isomorphism of lattices from an order isomorphism between them.
Equations
- Lat.Iso.mk e = { hom := { toFun := ⇑e, map_sup' := ⋯, map_inf' := ⋯ }, inv := { toFun := ⇑e.symm, map_sup' := ⋯, map_inf' := ⋯ }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
theorem
Lat.Iso.mk_hom_toSupHom_toFun
{α : Lat}
{β : Lat}
(e : ↑α ≃o ↑β)
(a : ↑α)
:
(Lat.Iso.mk e).hom.toSupHom a = e a
@[simp]
theorem
Lat.Iso.mk_inv_toSupHom_toFun
{α : Lat}
{β : Lat}
(e : ↑α ≃o ↑β)
(a : ↑β)
:
(Lat.Iso.mk e).inv.toSupHom a = e.symm a
OrderDual
as a functor.
Equations
- Lat.dual = { obj := fun (X : Lat) => Lat.of (↑X)ᵒᵈ, map := fun {X Y : Lat} => ⇑LatticeHom.dual, map_id := Lat.dual.proof_1, map_comp := @Lat.dual.proof_2 }
Instances For
@[simp]
theorem
Lat_dual_comp_forget_to_partOrd :
Lat.dual.comp (CategoryTheory.forget₂ Lat PartOrd) = (CategoryTheory.forget₂ Lat PartOrd).comp PartOrd.dual