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
Equations
- One or more equations did not get rendered due to their size.
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- SemiRingCat.Hom.Simps.hom R S f = f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- SemiRingCat.instInhabited = { default := SemiRingCat.of PUnit.{?u.3 + 1} }
This unification hint helps with problems of the form (forget ?C).obj R =?= carrier R'
.
Equations
- R.forget_obj_eq_coe R' = (R = R' → (CategoryTheory.forget SemiRingCat).obj R = ↑R')
Instances For
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.toSemiRingCatIso = { hom := SemiRingCat.ofHom ↑e, inv := SemiRingCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
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
Equations
- One or more equations did not get rendered due to their size.
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- RingCat.Hom.Simps.hom R S f = f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- RingCat.instInhabited = { default := RingCat.of PUnit.{?u.3 + 1} }
This unification hint helps with problems of the form (forget ?C).obj R =?= carrier R'
.
An example where this is needed is in applying
PresheafOfModules.Sheafify.app_eq_of_isLocallyInjective
.
Equations
- R.forget_obj_eq_coe R' = (R = R' → (CategoryTheory.forget RingCat).obj R = ↑R')
Instances For
Equations
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 := RingCat.ofHom ↑e, inv := RingCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The category of commutative 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
Equations
- One or more equations did not get rendered due to their size.
Typecheck a RingHom
as a morphism in CommSemiRingCat
.
Equations
Instances For
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- CommSemiRingCat.Hom.Simps.hom R S f = f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- CommSemiRingCat.instInhabited = { default := CommSemiRingCat.of PUnit.{?u.3 + 1} }
This unification hint helps with problems of the form (forget ?C).obj R =?= carrier R'
.
Equations
- R.forget_obj_eq_coe R' = (R = R' → (CategoryTheory.forget CommSemiRingCat).obj R = ↑R')
Instances For
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 := CommSemiRingCat.ofHom ↑e, inv := CommSemiRingCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The category of commutative rings.
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
Equations
- One or more equations did not get rendered due to their size.
The underlying ring hom.
Equations
Instances For
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- CommRingCat.Hom.Simps.hom R S f = f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- CommRingCat.instInhabited = { default := CommRingCat.of PUnit.{?u.3 + 1} }
This unification hint helps with problems of the form (forget ?C).obj R =?= carrier R'
.
An example where this is needed is in applying TopCat.Presheaf.restrictOpen
to commutative rings.
Equations
- R.forget_obj_eq_coe R' = (R = R' → (CategoryTheory.forget CommRingCat).obj R = ↑R')
Instances For
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
- One or more equations did not get rendered due to their size.
Ring equivalence are isomorphisms in category of semirings
Equations
- e.toCommRingCatIso = { hom := CommRingCat.ofHom ↑e, inv := CommRingCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build a RingEquiv
from an isomorphism in the category RingCat
.
Equations
- e.ringCatIsoToRingEquiv = RingEquiv.ofHomInv (RingCat.Hom.hom e.hom) (RingCat.Hom.hom e.inv) ⋯ ⋯
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.