mathlib3 documentation

order.category.BddDistLat

The category of bounded distributive lattices #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This defines BddDistLat, the category of bounded distributive lattices.

Note that this category is sometimes called DistLat when being a lattice is understood to entail having a bottom and a top element.

@[protected, instance]
Equations

Construct a bundled BddDistLat from a bounded_order distrib_lattice.

Equations
@[simp]
theorem BddDistLat.coe_of (α : Type u_1) [distrib_lattice α] [bounded_order α] :

Turn a BddDistLat into a BddLat by forgetting it is distributive.

Equations
@[protected, instance]
Equations
@[simp]
theorem BddDistLat.iso.mk_hom {α β : BddDistLat} (e : α ≃o β) :
def BddDistLat.iso.mk {α β : BddDistLat} (e : α ≃o β) :
α β

Constructs an equivalence between bounded distributive lattices from an order isomorphism between them.

Equations
@[simp]
theorem BddDistLat.iso.mk_inv {α β : BddDistLat} (e : α ≃o β) :

order_dual as a functor.

Equations