Documentation

Mathlib.AlgebraicGeometry.Morphisms.Constructors

Constructors for properties of morphisms between schemes #

This file provides some constructors to obtain morphism properties of schemes from other morphism properties:

Also provides API for showing the standard locality and stability properties for these types of properties.

The AffineTargetMorphismProperty associated to (targetAffineLocally P).diagonal. See diagonal_targetAffineLocally_eq_targetAffineLocally.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem AlgebraicGeometry.AffineTargetMorphismProperty.diagonal_respectsIso (P : AlgebraicGeometry.AffineTargetMorphismProperty) (hP : P.toProperty.RespectsIso) :
    P.diagonal.toProperty.RespectsIso
    theorem AlgebraicGeometry.diagonal_targetAffineLocally_of_openCover (P : AlgebraicGeometry.AffineTargetMorphismProperty) (hP : P.IsLocal) {X : AlgebraicGeometry.Scheme} {Y : AlgebraicGeometry.Scheme} (f : X Y) (𝒰 : Y.OpenCover) [∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)] (𝒰' : (i : 𝒰.J) → (CategoryTheory.Limits.pullback f (𝒰.map i)).OpenCover) [∀ (i : 𝒰.J) (j : (𝒰' i).J), AlgebraicGeometry.IsAffine ((𝒰' i).obj j)] (h𝒰' : ∀ (i : 𝒰.J) (j k : (𝒰' i).J), P (CategoryTheory.Limits.pullback.mapDesc ((𝒰' i).map j) ((𝒰' i).map k) CategoryTheory.Limits.pullback.snd)) :
    theorem AlgebraicGeometry.AffineTargetMorphismProperty.IsLocal.diagonal_affine_openCover_TFAE {P : AlgebraicGeometry.AffineTargetMorphismProperty} (hP : P.IsLocal) {X : AlgebraicGeometry.Scheme} {Y : AlgebraicGeometry.Scheme} (f : X Y) :
    [(AlgebraicGeometry.targetAffineLocally P).diagonal f, ∃ (𝒰 : Y.OpenCover) (x : ∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)), ∀ (i : 𝒰.J), P.diagonal CategoryTheory.Limits.pullback.snd, ∀ (𝒰 : Y.OpenCover) [inst : ∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)] (i : 𝒰.J), P.diagonal CategoryTheory.Limits.pullback.snd, ∀ {U : AlgebraicGeometry.Scheme} (g : U Y) [inst : AlgebraicGeometry.IsAffine U] [inst_1 : AlgebraicGeometry.IsOpenImmersion g], P.diagonal CategoryTheory.Limits.pullback.snd, ∃ (𝒰 : Y.OpenCover) (x : ∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)) (𝒰' : (i : 𝒰.J) → (CategoryTheory.Limits.pullback f (𝒰.map i)).OpenCover) (x_1 : ∀ (i : 𝒰.J) (j : (𝒰' i).J), AlgebraicGeometry.IsAffine ((𝒰' i).obj j)), ∀ (i : 𝒰.J) (j k : (𝒰' i).J), P (CategoryTheory.Limits.pullback.mapDesc ((𝒰' i).map j) ((𝒰' i).map k) CategoryTheory.Limits.pullback.snd)].TFAE
    theorem AlgebraicGeometry.universally_isLocalAtTarget (P : CategoryTheory.MorphismProperty AlgebraicGeometry.Scheme) (hP : ∀ {X Y : AlgebraicGeometry.Scheme} (f : X Y) (𝒰 : Y.OpenCover), (∀ (i : 𝒰.J), P CategoryTheory.Limits.pullback.snd)P f) :
    theorem AlgebraicGeometry.universally_isLocalAtTarget_of_morphismRestrict (P : CategoryTheory.MorphismProperty AlgebraicGeometry.Scheme) (hP₁ : P.RespectsIso) (hP₂ : ∀ {X Y : AlgebraicGeometry.Scheme} (f : X Y) {ι : Type u} (U : ιTopologicalSpace.Opens Y.toPresheafedSpace), iSup U = (∀ (i : ι), P (f ∣_ U i))P f) :

    topologically P holds for a morphism if the underlying topological map satisfies P.

    Equations
    Instances For
      theorem AlgebraicGeometry.MorphismProperty.topologically_isStableUnderComposition (P : {α β : Type u} → [inst : TopologicalSpace α] → [inst : TopologicalSpace β] → (αβ)Prop) (hP : ∀ {α β γ : Type u} [inst : TopologicalSpace α] [inst_1 : TopologicalSpace β] [inst_2 : TopologicalSpace γ] (f : αβ) (g : βγ), P fP gP (g f)) :
      (AlgebraicGeometry.MorphismProperty.topologically fun {α β : Type u} [TopologicalSpace α] [TopologicalSpace β] => P).IsStableUnderComposition

      If a property of maps of topological spaces is stable under composition, the induced morphism property of schemes is stable under composition.

      If a property of maps of topological spaces is satisfied by all homeomorphisms, every isomorphism of schemes satisfies the induced property.

      theorem AlgebraicGeometry.MorphismProperty.topologically_respectsIso (P : {α β : Type u} → [inst : TopologicalSpace α] → [inst : TopologicalSpace β] → (αβ)Prop) (hP₁ : ∀ {α β : Type u} [inst : TopologicalSpace α] [inst_1 : TopologicalSpace β] (f : α ≃ₜ β), P f) (hP₂ : ∀ {α β γ : Type u} [inst : TopologicalSpace α] [inst_1 : TopologicalSpace β] [inst_2 : TopologicalSpace γ] (f : αβ) (g : βγ), P fP gP (g f)) :

      If a property of maps of topological spaces is satisfied by homeomorphisms and is stable under composition, the induced property on schemes respects isomorphisms.

      theorem AlgebraicGeometry.MorphismProperty.topologically_propertyIsLocalAtTarget (P : {α β : Type u} → [inst : TopologicalSpace α] → [inst : TopologicalSpace β] → (αβ)Prop) (hP₁ : (AlgebraicGeometry.MorphismProperty.topologically fun {α β : Type u} [TopologicalSpace α] [TopologicalSpace β] => P).RespectsIso) (hP₂ : ∀ {α β : Type u} [inst : TopologicalSpace α] [inst_1 : TopologicalSpace β] (f : αβ) (s : Set β), P fP (s.restrictPreimage f)) (hP₃ : ∀ {α β : Type u} [inst : TopologicalSpace α] [inst_1 : TopologicalSpace β] (f : αβ) {ι : Type u} (U : ιTopologicalSpace.Opens β), iSup U = Continuous f(∀ (i : ι), P ((U i).carrier.restrictPreimage f))P f) :

      To check that a topologically defined morphism property is local at the target, we may check the corresponding properties on topological spaces.

      @[deprecated AlgebraicGeometry.diagonal_targetAffineLocally_of_openCover]
      theorem AlgebraicGeometry.diagonalTargetAffineLocallyOfOpenCover (P : AlgebraicGeometry.AffineTargetMorphismProperty) (hP : P.IsLocal) {X : AlgebraicGeometry.Scheme} {Y : AlgebraicGeometry.Scheme} (f : X Y) (𝒰 : Y.OpenCover) [∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)] (𝒰' : (i : 𝒰.J) → (CategoryTheory.Limits.pullback f (𝒰.map i)).OpenCover) [∀ (i : 𝒰.J) (j : (𝒰' i).J), AlgebraicGeometry.IsAffine ((𝒰' i).obj j)] (h𝒰' : ∀ (i : 𝒰.J) (j k : (𝒰' i).J), P (CategoryTheory.Limits.pullback.mapDesc ((𝒰' i).map j) ((𝒰' i).map k) CategoryTheory.Limits.pullback.snd)) :

      Alias of AlgebraicGeometry.diagonal_targetAffineLocally_of_openCover.

      @[deprecated AlgebraicGeometry.AffineTargetMorphismProperty.diagonal_of_targetAffineLocally]

      Alias of AlgebraicGeometry.AffineTargetMorphismProperty.diagonal_of_targetAffineLocally.

      @[deprecated AlgebraicGeometry.universally_isLocalAtTarget]
      theorem AlgebraicGeometry.universallyIsLocalAtTarget (P : CategoryTheory.MorphismProperty AlgebraicGeometry.Scheme) (hP : ∀ {X Y : AlgebraicGeometry.Scheme} (f : X Y) (𝒰 : Y.OpenCover), (∀ (i : 𝒰.J), P CategoryTheory.Limits.pullback.snd)P f) :

      Alias of AlgebraicGeometry.universally_isLocalAtTarget.

      @[deprecated AlgebraicGeometry.universally_isLocalAtTarget_of_morphismRestrict]
      theorem AlgebraicGeometry.universallyIsLocalAtTargetOfMorphismRestrict (P : CategoryTheory.MorphismProperty AlgebraicGeometry.Scheme) (hP₁ : P.RespectsIso) (hP₂ : ∀ {X Y : AlgebraicGeometry.Scheme} (f : X Y) {ι : Type u} (U : ιTopologicalSpace.Opens Y.toPresheafedSpace), iSup U = (∀ (i : ι), P (f ∣_ U i))P f) :

      Alias of AlgebraicGeometry.universally_isLocalAtTarget_of_morphismRestrict.