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.
- carrier : Type u
The underlying type.
- booleanRing : BooleanRing ↑self
Instances For
Equations
- BoolRing.instCoeSortType = { coe := BoolRing.carrier }
@[reducible, inline]
Construct a bundled BoolRing
from a BooleanRing
.
Equations
- BoolRing.of α = BoolRing.mk✝ α
Instances For
Equations
- BoolRing.instInhabited = { default := BoolRing.of PUnit.{?u.3 + 1} }
instance
BoolRing.instConcreteCategoryRingHomCarrier :
CategoryTheory.ConcreteCategory BoolRing fun (x1 x2 : BoolRing) => ↑x1 →+* ↑x2
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.
Constructs an isomorphism of Boolean rings from a ring isomorphism between them.
Equations
- BoolRing.Iso.mk e = { hom := { hom' := ↑e }, inv := { hom' := ↑e.symm }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
@[simp]
@[simp]
Equations
- One or more equations did not get rendered due to their size.
@[simp]
@[simp]
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.