The category of finite Boolean algebras #
This file defines FinBoolAlg, the category of finite Boolean algebras.
TODO #
Birkhoff's representation for finite Boolean algebras.
FintypeCat_to_FinBoolAlg_op.left_op ⋙ FinBoolAlg.dual ≅
FintypeCat_to_FinBoolAlg_op.left_op
FinBoolAlg is essentially small.
Equations
- FinBoolAlg.instCoeSortType = { coe := fun (X : FinBoolAlg) => ↑X.toBoolAlg }
@[reducible, inline]
Construct a bundled FinBoolAlg from BooleanAlgebra + Fintype.
Equations
- FinBoolAlg.of α = { carrier := α, str := inst✝¹, isFintype := inst✝ }
Instances For
Equations
- FinBoolAlg.instInhabited = { default := FinBoolAlg.of PUnit.{?u.2 + 1} }
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]
@[simp]
@[simp]
Constructs an equivalence between finite Boolean algebras from an order isomorphism between them.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
theorem
FinBoolAlg.Iso.mk_hom
{α β : FinBoolAlg}
(e : ↑α.toBoolAlg ≃o ↑β.toBoolAlg)
:
(mk e).hom = CategoryTheory.InducedCategory.homMk
(BoolAlg.ofHom
(have __src := { toFun := ⇑e, map_sup' := ⋯, map_inf' := ⋯ };
{ toFun := ⇑e, map_sup' := ⋯, map_inf' := ⋯, map_top' := ⋯, map_bot' := ⋯ }))
OrderDual as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
The equivalence between FinBoolAlg and itself induced by OrderDual both ways.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The powerset functor. Set as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
theorem
fintypeToFinBoolAlgOp_map
{X Y : FintypeCat}
(f : X ⟶ Y)
:
fintypeToFinBoolAlgOp.map f = (CategoryTheory.InducedCategory.homMk
(BoolAlg.ofHom
(have __src :=
{ toFun := ⇑(CompleteLatticeHom.setPreimage ⇑(CategoryTheory.ConcreteCategory.hom f)), map_sup' := ⋯,
map_inf' := ⋯ };
{ toFun := ⇑(CompleteLatticeHom.setPreimage ⇑(CategoryTheory.ConcreteCategory.hom f)), map_sup' := ⋯,
map_inf' := ⋯, map_top' := ⋯, map_bot' := ⋯ }))).op