Ring-theoretic results in terms of categorical languages #
instance
localization_unit_isIso
(R : CommRingCat)
:
CategoryTheory.IsIso (CommRingCat.ofHom (algebraMap (↑R) (Localization.Away 1)))
instance
localization_unit_isIso'
(R : CommRingCat)
:
CategoryTheory.IsIso (CommRingCat.ofHom (algebraMap (↑R) (Localization.Away 1)))
theorem
IsLocalization.epi
{R : Type u_1}
[CommRing R]
(M : Submonoid R)
(S : Type u_1)
[CommRing S]
[Algebra R S]
[IsLocalization M S]
:
instance
Localization.epi'
{R : CommRingCat}
(M : Submonoid ↑R)
:
CategoryTheory.Epi (CommRingCat.ofHom (algebraMap (↑R) (Localization M)))
instance
CommRingCat.isLocalHom_comp
{R S T : CommRingCat}
(f : R ⟶ S)
(g : S ⟶ T)
[IsLocalHom g.hom]
[IsLocalHom f.hom]
:
IsLocalHom (CategoryTheory.CategoryStruct.comp f g).hom
@[deprecated CommRingCat.isLocalHom_comp]
theorem
CommRingCat.isLocalRingHom_comp
{R S T : CommRingCat}
(f : R ⟶ S)
(g : S ⟶ T)
[IsLocalHom g.hom]
[IsLocalHom f.hom]
:
IsLocalHom (CategoryTheory.CategoryStruct.comp f g).hom
Alias of CommRingCat.isLocalHom_comp
.
@[deprecated isLocalHom_of_iso]
Alias of isLocalHom_of_iso
.
@[instance 100]
instance
isLocalHom_of_isIso
{R S : CommRingCat}
(f : R ⟶ S)
[CategoryTheory.IsIso f]
:
IsLocalHom f.hom
@[deprecated isLocalHom_of_isIso]
theorem
isLocalRingHom_of_isIso
{R S : CommRingCat}
(f : R ⟶ S)
[CategoryTheory.IsIso f]
:
IsLocalHom f.hom
Alias of isLocalHom_of_isIso
.