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 (Hom.hom g)]
[IsLocalHom (Hom.hom f)]
:
@[deprecated CommRingCat.isLocalHom_comp (since := "2024-10-10")]
theorem
CommRingCat.isLocalRingHom_comp
{R S T : CommRingCat}
(f : R ⟶ S)
(g : S ⟶ T)
[IsLocalHom (Hom.hom g)]
[IsLocalHom (Hom.hom f)]
:
Alias of CommRingCat.isLocalHom_comp
.
@[deprecated isLocalHom_of_iso (since := "2024-10-10")]
Alias of isLocalHom_of_iso
.
@[instance 100]
@[deprecated isLocalHom_of_isIso (since := "2024-10-10")]
Alias of isLocalHom_of_isIso
.