Properties of morphisms from properties of ring homs. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We provide the basic framework for talking about properties of morphisms that come from properties
of ring homs. For P
a property of ring homs, we have two ways of defining a property of scheme
morphisms:
Let f : X ⟶ Y
,
target_affine_locally (affine_and P)
: the preimage of an affine openU = Spec A
is affine (= Spec B
) andA ⟶ B
satisfiesP
. (TODO)affine_locally P
: For each pair of affine openU = Spec A ⊆ X
andV = Spec B ⊆ f ⁻¹' U
, the ring homA ⟶ B
satisfiesP
.
For these notions to be well defined, we require P
be a sufficient local property. For the former,
P
should be local on the source (ring_hom.respects_iso P
, ring_hom.localization_preserves P
,
ring_hom.of_localization_span
), and target_affine_locally (affine_and P)
will be local on
the target. (TODO)
For the latter P
should be local on the target (ring_hom.property_is_local P
), and
affine_locally P
will be local on both the source and the target.
Further more, these properties are stable under compositions (resp. base change) if P
is. (TODO)
For P
a property of ring homomorphisms, source_affine_locally P
holds for f : X ⟶ Y
whenever P
holds for the restriction of f
on every affine open subset of X
.
Equations
- algebraic_geometry.source_affine_locally P = λ (X Y : algebraic_geometry.Scheme) (f : X ⟶ Y) (hY : algebraic_geometry.is_affine Y), ∀ (U : ↥(X.affine_opens)), P (algebraic_geometry.Scheme.Γ.map (X.of_restrict _ ≫ f).op)
For P
a property of ring homomorphisms, affine_locally P
holds for f : X ⟶ Y
if for each
affine open U = Spec A ⊆ Y
and V = Spec B ⊆ f ⁻¹' U
, the ring hom A ⟶ B
satisfies P
.
Also see affine_locally_iff_affine_opens_le
.