Category instances for Semiring
, Ring
, CommSemiring
, and CommRing
. #
We introduce the bundled categories:
SemiRingCat
RingCat
CommSemiRingCat
CommRingCat
along with the relevant forgetful functors between them.
The category of semirings.
Instances For
Equations
- SemiRingCat.instCoeSortType = { coe := SemiRingCat.carrier }
The object in the category of R-algebras associated to a type equipped with the appropriate
typeclasses. This is the preferred way to construct a term of SemiRingCat
.
Equations
Instances For
Typecheck a RingHom
as a morphism in SemiRingCat
.
Equations
- SemiRingCat.ofHom f = { hom := f }
Instances For
Equations
- SemiRingCat.instInhabited = { default := SemiRingCat.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Equations
- SemiRingCat.instSemiringObjForget = inferInstance
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.
Equations
- RingCat.instCoeSortType = { coe := RingCat.carrier }
The object in the category of R-algebras associated to a type equipped with the appropriate
typeclasses. This is the preferred way to construct a term of RingCat
.
Equations
- RingCat.of R = RingCat.mk✝ R
Instances For
Typecheck a RingHom
as a morphism in RingCat
.
Equations
- RingCat.ofHom f = { hom := f }
Instances For
Equations
- RingCat.instInhabited = { default := RingCat.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Equations
- RingCat.instRingObjForget = inferInstance
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.
Ring equivalence are isomorphisms in category of semirings
Equations
- e.toRingCatIso = { hom := { hom := ↑e }, inv := { hom := ↑e.symm }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The category of semirings.
- carrier : Type u
The underlying type.
- commSemiring : CommSemiring ↑self
Instances For
Equations
The object in the category of R-algebras associated to a type equipped with the appropriate
typeclasses. This is the preferred way to construct a term of CommSemiRingCat
.
Equations
Instances For
Typecheck a RingHom
as a morphism in CommSemiRingCat
.
Equations
- CommSemiRingCat.ofHom f = { hom := f }
Instances For
Equations
- CommSemiRingCat.instInhabited = { default := CommSemiRingCat.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Equations
- CommSemiRingCat.instCommSemiringObjForget = inferInstance
Equations
- One or more equations did not get rendered due to their size.
The forgetful functor from commutative rings to (multiplicative) commutative monoids.
Equations
- One or more equations did not get rendered due to their size.
Ring equivalence are isomorphisms in category of semirings
Equations
- e.toCommSemiRingCatIso = { hom := { hom := ↑e }, inv := { hom := ↑e.symm }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The category of semirings.
Instances For
Equations
- CommRingCat.instCoeSortType = { coe := CommRingCat.carrier }
The object in the category of R-algebras associated to a type equipped with the appropriate
typeclasses. This is the preferred way to construct a term of CommRingCat
.
Equations
Instances For
Typecheck a RingHom
as a morphism in CommRingCat
.
Equations
- CommRingCat.ofHom f = { hom := f }
Instances For
Equations
- CommRingCat.instInhabited = { default := CommRingCat.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Equations
- CommRingCat.instCommRingObjForget = inferInstance
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.
Build a RingEquiv
from an isomorphism in the category SemiRingCat
.
Equations
- e.semiRingCatIsoToRingEquiv = RingEquiv.ofHomInv e.hom.hom e.inv.hom ⋯ ⋯
Instances For
Build a RingEquiv
from an isomorphism in the category RingCat
.
Equations
- e.ringCatIsoToRingEquiv = RingEquiv.ofHomInv e.hom.hom e.inv.hom ⋯ ⋯
Instances For
Build a RingEquiv
from an isomorphism in the category CommSemiRingCat
.
Equations
- e.commSemiRingCatIsoToRingEquiv = RingEquiv.ofHomInv e.hom.hom e.inv.hom ⋯ ⋯
Instances For
Build a RingEquiv
from an isomorphism in the category CommRingCat
.
Equations
- e.commRingCatIsoToRingEquiv = RingEquiv.ofHomInv e.hom.hom e.inv.hom ⋯ ⋯
Instances For
An alias for SemiringCat.{max u v}
, to deal around unification issues.
Equations
Instances For
An alias for RingCat.{max u v}
, to deal around unification issues.
Equations
Instances For
An alias for CommSemiRingCat.{max u v}
, to deal around unification issues.
Equations
Instances For
An alias for CommRingCat.{max u v}
, to deal around unification issues.