Documentation

Mathlib.Algebra.Category.Ring.Instances

Ring-theoretic results in terms of categorical languages #

@[deprecated CommRingCat.isLocalHom_comp]

Alias of CommRingCat.isLocalHom_comp.

theorem isLocalHom_of_iso {R S : CommRingCat} (f : R S) :
IsLocalHom f.hom.hom
@[deprecated isLocalHom_of_iso]
theorem isLocalRingHom_of_iso {R S : CommRingCat} (f : R S) :
IsLocalHom f.hom.hom

Alias of isLocalHom_of_iso.

@[instance 100]
instance isLocalHom_of_isIso {R S : CommRingCat} (f : R S) [CategoryTheory.IsIso f] :
@[deprecated isLocalHom_of_isIso]

Alias of isLocalHom_of_isIso.