The category of bounded lattices #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines BddLat
, the category of bounded lattices.
In literature, this is sometimes called Lat
, the category of lattices, because being a lattice is
understood to entail having a bottom and a top element.
- to_Lat : Lat
- is_bounded_order : bounded_order ↥(self.to_Lat)
The category of bounded lattices with bounded lattice morphisms.
Instances for BddLat
- BddLat.has_sizeof_inst
- BddLat.has_coe_to_sort
- BddLat.inhabited
- BddLat.category_theory.large_category
- BddLat.category_theory.concrete_category
- BddLat.has_forget_to_BddOrd
- BddLat.has_forget_to_Lat
- BddLat.has_forget_to_SemilatSup
- BddLat.has_forget_to_SemilatInf
- BddDistLat.has_forget_to_BddLat
- CompleteLat.has_forget_to_BddLat
Equations
Equations
- BddLat.category_theory.large_category = {to_category_struct := {to_quiver := {hom := λ (X Y : BddLat), bounded_lattice_hom ↥X ↥Y}, id := λ (X : BddLat), bounded_lattice_hom.id ↥X, comp := λ (X Y Z : BddLat) (f : X ⟶ Y) (g : Y ⟶ Z), bounded_lattice_hom.comp g f}, id_comp' := BddLat.category_theory.large_category._proof_1, comp_id' := BddLat.category_theory.large_category._proof_2, assoc' := BddLat.category_theory.large_category._proof_3}
Equations
- BddLat.category_theory.concrete_category = category_theory.concrete_category.mk {obj := coe_sort BddLat.has_coe_to_sort, map := λ (X Y : BddLat), coe_fn, map_id' := BddLat.category_theory.concrete_category._proof_1, map_comp' := BddLat.category_theory.concrete_category._proof_2}
Equations
- BddLat.has_forget_to_BddOrd = {forget₂ := {obj := λ (X : BddLat), BddOrd.of ↥X, map := λ (X Y : BddLat), bounded_lattice_hom.to_bounded_order_hom, map_id' := BddLat.has_forget_to_BddOrd._proof_1, map_comp' := BddLat.has_forget_to_BddOrd._proof_2}, forget_comp := BddLat.has_forget_to_BddOrd._proof_3}
Equations
Equations
- BddLat.has_forget_to_SemilatSup = {forget₂ := {obj := λ (X : BddLat), SemilatSup.mk ↥X, map := λ (X Y : BddLat), bounded_lattice_hom.to_sup_bot_hom, map_id' := BddLat.has_forget_to_SemilatSup._proof_1, map_comp' := BddLat.has_forget_to_SemilatSup._proof_2}, forget_comp := BddLat.has_forget_to_SemilatSup._proof_3}
Equations
- BddLat.has_forget_to_SemilatInf = {forget₂ := {obj := λ (X : BddLat), SemilatInf.mk ↥X, map := λ (X Y : BddLat), bounded_lattice_hom.to_inf_top_hom, map_id' := BddLat.has_forget_to_SemilatInf._proof_1, map_comp' := BddLat.has_forget_to_SemilatInf._proof_2}, forget_comp := BddLat.has_forget_to_SemilatInf._proof_3}
Constructs an equivalence between bounded lattices from an order isomorphism between them.
Equations
- BddLat.iso.mk e = {hom := ↑e, inv := ↑(e.symm), hom_inv_id' := _, inv_hom_id' := _}
order_dual
as a functor.
The equivalence between BddLat
and itself induced by order_dual
both ways.
Equations
- BddLat.dual_equiv = category_theory.equivalence.mk BddLat.dual BddLat.dual (category_theory.nat_iso.of_components (λ (X : BddLat), BddLat.iso.mk (order_iso.dual_dual ↥X)) BddLat.dual_equiv._proof_1) (category_theory.nat_iso.of_components (λ (X : BddLat), BddLat.iso.mk (order_iso.dual_dual ↥X)) BddLat.dual_equiv._proof_2)
The functor that adds a bottom and a top element to a lattice. This is the free functor.
Lat_to_BddLat
is left adjoint to the forgetful functor, meaning it is the free
functor from Lat
to BddLat
.
Equations
- Lat_to_BddLat_forget_adjunction = category_theory.adjunction.mk_of_hom_equiv {hom_equiv := λ (X : Lat) (Y : BddLat), {to_fun := λ (f : Lat_to_BddLat.obj X ⟶ Y), {to_sup_hom := {to_fun := ⇑f ∘ option.some ∘ option.some, map_sup' := _}, map_inf' := _}, inv_fun := lattice_hom.with_top_with_bot' Y.is_bounded_order, left_inv := _, right_inv := _}, hom_equiv_naturality_left_symm' := Lat_to_BddLat_forget_adjunction._proof_5, hom_equiv_naturality_right' := Lat_to_BddLat_forget_adjunction._proof_6}
Lat_to_BddLat
and order_dual
commute.