Documentation

Mathlib.AlgebraicGeometry.Properties

Basic properties of schemes #

We provide some basic properties of schemes

Main definition #

A scheme X is reduced if all 𝒪ₓ(U) are reduced.

Instances
    theorem AlgebraicGeometry.isReduced_of_isReduced_stalk (X : Scheme) [∀ (x : X.toPresheafedSpace), _root_.IsReduced (X.presheaf.stalk x)] :
    instance AlgebraicGeometry.isReduced_stalk_of_isReduced (X : Scheme) [IsReduced X] (x : X.toPresheafedSpace) :
    _root_.IsReduced (X.presheaf.stalk x)
    theorem AlgebraicGeometry.reduce_to_affine_global (P : {X : Scheme} → X.OpensProp) {X : Scheme} (U : X.Opens) (h₁ : ∀ (X : Scheme) (U : X.Opens), (∀ (x : U), ∃ (V : X.Opens) (_ : x V) (x : V U), P V)P U) (h₂ : ∀ (X Y : Scheme) (f : X Y) [inst : IsOpenImmersion f], ∃ (U : X.Opens) (V : Y.Opens), U = V = Scheme.Hom.opensRange f (P UP V)) (h₃ : ∀ (R : CommRingCat), P ) :
    P U

    To show that a statement P holds for all open subsets of all schemes, it suffices to show that

    1. In any scheme X, if P holds for an open cover of U, then P holds for U.
    2. For an open immerison f : X ⟶ Y, if P holds for the entire space of X, then P holds for the image of f.
    3. P holds for the entire space of an affine scheme.
    theorem AlgebraicGeometry.reduce_to_affine_nbhd (P : (X : Scheme) → X.toPresheafedSpaceProp) (h₁ : ∀ (R : CommRingCat) (x : (Spec R).toPresheafedSpace), P (Spec R) x) (h₂ : ∀ {X Y : Scheme} (f : X Y) [inst : IsOpenImmersion f] (x : X.toPresheafedSpace), P X xP Y (f.base x)) (X : Scheme) (x : X.toPresheafedSpace) :
    P X x
    theorem AlgebraicGeometry.eq_zero_of_basicOpen_eq_bot {X : Scheme} [hX : IsReduced X] {U : X.Opens} (s : (X.presheaf.obj (Opposite.op U))) (hs : X.basicOpen s = ) :
    s = 0
    @[simp]
    theorem AlgebraicGeometry.basicOpen_eq_bot_iff {X : Scheme} [IsReduced X] {U : X.Opens} (s : (X.presheaf.obj (Opposite.op U))) :
    X.basicOpen s = s = 0

    A scheme X is integral if its is nonempty, and 𝒪ₓ(U) is an integral domain for each U ≠ ∅.

    Instances
      instance AlgebraicGeometry.Scheme.component_nontrivial (X : Scheme) (U : X.Opens) [Nonempty (↑U).toPresheafedSpace] :
      Nontrivial (X.presheaf.obj (Opposite.op U))
      theorem AlgebraicGeometry.isIntegral_of_isOpenImmersion {X Y : Scheme} (f : X Y) [H : IsOpenImmersion f] [IsIntegral Y] [Nonempty X.toPresheafedSpace] :
      theorem AlgebraicGeometry.isIntegral_of_isAffine_of_isDomain (X : Scheme) [IsAffine X] [Nonempty X.toPresheafedSpace] [IsDomain (X.presheaf.obj (Opposite.op ))] :
      theorem AlgebraicGeometry.map_injective_of_isIntegral (X : Scheme) [IsIntegral X] {U V : X.Opens} (i : U V) [H : Nonempty (↑U).toPresheafedSpace] :
      Function.Injective (X.presheaf.map i.op).hom