The category of distributive lattices #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines DistLat
, the category of distributive lattices.
Note that DistLat
in the literature doesn't always
correspond to DistLat
as we don't require bottom or top elements. Instead, this DistLat
corresponds to BddDistLat
.
The category of distributive lattices.
Equations
@[protected, instance]
@[protected, instance]
Equations
- X.distrib_lattice = X.str
Construct a bundled DistLat
from a distrib_lattice
underlying type and typeclass.
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
- DistLat.distrib_lattice.to_lattice.category_theory.bundled_hom.parent_projection = category_theory.bundled_hom.parent_projection.mk
@[protected, instance]
@[protected, instance]
@[simp]
Constructs an equivalence between distributive lattices from an order isomorphism between them.
Equations
- DistLat.iso.mk e = {hom := ↑e, inv := ↑(e.symm), hom_inv_id' := _, inv_hom_id' := _}
@[simp]
order_dual
as a functor.
Equations
- DistLat.dual = {obj := λ (X : DistLat), DistLat.of (↥X)ᵒᵈ, map := λ (X Y : DistLat), ⇑lattice_hom.dual, map_id' := DistLat.dual._proof_1, map_comp' := DistLat.dual._proof_2}
The equivalence between DistLat
and itself induced by order_dual
both ways.
Equations
- DistLat.dual_equiv = category_theory.equivalence.mk DistLat.dual DistLat.dual (category_theory.nat_iso.of_components (λ (X : DistLat), DistLat.iso.mk (order_iso.dual_dual ↥X)) DistLat.dual_equiv._proof_1) (category_theory.nat_iso.of_components (λ (X : DistLat), DistLat.iso.mk (order_iso.dual_dual ↥X)) DistLat.dual_equiv._proof_2)