Properties of ring homomorphisms #
We provide the basic framework for talking about properties of ring homomorphisms. The following meta-properties of predicates on ring homomorphisms are defined
RingHom.RespectsIso
:P
respects isomorphisms ifP f → P (e ≫ f)
andP f → P (f ≫ e)
, wheree
is an isomorphism.RingHom.StableUnderComposition
:P
is stable under composition ifP f → P g → P (f ≫ g)
.RingHom.IsStableUnderBaseChange
:P
is stable under base change ifP (S ⟶ Y)
impliesP (X ⟶ X ⊗[S] Y)
.
def
RingHom.RespectsIso
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
:
A property RespectsIso
if it still holds when composed with an isomorphism
Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
RingHom.RespectsIso.cancel_left_isIso
{P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop}
(hP : RespectsIso P)
{R S T : CommRingCat}
(f : R ⟶ S)
(g : S ⟶ T)
[CategoryTheory.IsIso f]
:
theorem
RingHom.RespectsIso.cancel_right_isIso
{P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop}
(hP : RespectsIso P)
{R S T : CommRingCat}
(f : R ⟶ S)
(g : S ⟶ T)
[CategoryTheory.IsIso g]
:
theorem
RingHom.RespectsIso.is_localization_away_iff
{P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop}
(hP : RespectsIso P)
{R S : Type u}
(R' S' : Type u)
[CommRing R]
[CommRing S]
[CommRing R']
[CommRing S']
[Algebra R R']
[Algebra S S']
(f : R →+* S)
(r : R)
[IsLocalization.Away r R']
[IsLocalization.Away (f r) S']
:
def
RingHom.StableUnderComposition
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
:
A property is StableUnderComposition
if the composition of two such morphisms
still falls in the class.
Equations
Instances For
def
RingHom.IsStableUnderBaseChange
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
:
A morphism property P
is IsStableUnderBaseChange
if P(S →+* A)
implies
P(B →+* A ⊗[S] B)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
RingHom.IsStableUnderBaseChange.mk
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
(h₁ : RespectsIso P)
(h₂ :
∀ ⦃R S T : Type u⦄ [inst : CommRing R] [inst_1 : CommRing S] [inst_2 : CommRing T] [inst_3 : Algebra R S]
[inst_4 : Algebra R T], P (algebraMap R T) → P Algebra.TensorProduct.includeLeftRingHom)
:
theorem
RingHom.IsStableUnderBaseChange.pushout_inl
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
(hP : IsStableUnderBaseChange P)
(hP' : RespectsIso P)
{R S T : CommRingCat}
(f : R ⟶ S)
(g : R ⟶ T)
(H : P (CommRingCat.Hom.hom g))
:
def
RingHom.toMorphismProperty
(P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop)
:
The categorical MorphismProperty
associated to a property of ring homs expressed
non-categorical terms.
Equations
- RingHom.toMorphismProperty P f = P (CommRingCat.Hom.hom f)
Instances For
theorem
RingHom.toMorphismProperty_respectsIso_iff
{P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop}
:
(RespectsIso fun {R S : Type u} [CommRing R] [CommRing S] => P) ↔ (toMorphismProperty fun {R S : Type u} [CommRing R] [CommRing S] => P).RespectsIso
theorem
RingHom.RespectsIso.arrow_mk_iso_iff
{P : {R S : Type u} → [inst : CommRing R] → [inst_1 : CommRing S] → (R →+* S) → Prop}
(hQ : RespectsIso fun {R S : Type u} [CommRing R] [CommRing S] => P)
{A B A' B' : CommRingCat}
{f : A ⟶ B}
{g : A' ⟶ B'}
(e : CategoryTheory.Arrow.mk f ≅ CategoryTheory.Arrow.mk g)
:
Variant of MorphismProperty.arrow_mk_iso_iff
specialized to morphism properties in
CommRingCat
given by ring hom properties.