The category of Boolean rings #
This file defines BoolRing
, the category of Boolean rings.
TODO #
Finish the equivalence with BoolAlg
.
The category of Boolean rings.
Equations
Instances For
Equations
- BoolRing.instCoeSortType = CategoryTheory.Bundled.coeSort
Equations
- X.instBooleanRingα = X.str
Equations
- BoolRing.instInhabited = { default := BoolRing.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Equations
- BoolRing.instConcreteCategory = id inferInstance
Equations
- One or more equations did not get rendered due to their size.
Constructs an isomorphism of Boolean rings from a ring isomorphism between them.
Equations
- BoolRing.Iso.mk e = { hom := ↑e, inv := ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
@[simp]
Equations
- One or more equations did not get rendered due to their size.
@[simp]
theorem
BoolRing.hasForgetToBoolAlg_forget₂_obj
(X : BoolRing)
:
CategoryTheory.HasForget₂.forget₂.obj X = BoolAlg.of (AsBoolAlg ↑X)
@[simp]
theorem
BoolRing.hasForgetToBoolAlg_forget₂_map
{x✝ x✝¹ : BoolRing}
(f : ↑x✝ →+* ↑x✝¹)
:
CategoryTheory.HasForget₂.forget₂.map f = f.asBoolAlg
instance
instBooleanAlgebraαLatticeToLatToBddLatToBddDistLat
{X : BoolAlg}
:
BooleanAlgebra ↑X.toBddDistLat.toBddLat.toLat
Equations
- instBooleanAlgebraαLatticeToLatToBddLatToBddDistLat = X.instBooleanAlgebra
Equations
- One or more equations did not get rendered due to their size.
@[simp]
theorem
BoolAlg.hasForgetToBoolRing_forget₂_obj
(X : BoolAlg)
:
CategoryTheory.HasForget₂.forget₂.obj X = BoolRing.of (AsBoolRing ↑X)
@[simp]
theorem
BoolAlg.hasForgetToBoolRing_forget₂_map
{x✝ x✝¹ : BoolAlg}
(f : BoundedLatticeHom ↑x✝.toBddDistLat.toBddLat.toLat ↑x✝¹.toBddDistLat.toBddLat.toLat)
:
CategoryTheory.HasForget₂.forget₂.map f = f.asBoolRing
The equivalence between Boolean rings and Boolean algebras. This is actually an isomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]