Documentation

Mathlib.AlgebraicGeometry.Noetherian

Noetherian and Locally Noetherian Schemes #

We introduce the concept of (locally) Noetherian schemes, giving definitions, equivalent conditions, and basic properties.

Main definitions #

Main results #

References #

A scheme X is locally Noetherian if 𝒪ₓ(U) is Noetherian for all affine U.

Instances
    theorem AlgebraicGeometry.isNoetherianRing_of_away {R : Type u} [CommRing R] (S : Finset R) (hS : Ideal.span S = ) (hN : ∀ (s : { x : R // x S }), IsNoetherianRing (Localization.Away s)) :

    Let R be a ring, and f i a finite collection of elements of R generating the unit ideal. If the localization of R at each f i is noetherian, so is R.

    We follow the proof given in [Har77], Proposition II.3.2

    theorem AlgebraicGeometry.isLocallyNoetherian_of_affine_cover {X : AlgebraicGeometry.Scheme} {ι : Sort u_1} {S : ιX.affineOpens} (hS : ⨆ (i : ι), (S i) = ) (hS' : ∀ (i : ι), IsNoetherianRing (X.presheaf.obj (Opposite.op (S i)))) :

    If a scheme X has a cover by affine opens whose sections are Noetherian rings, then X is locally Noetherian.

    theorem AlgebraicGeometry.isLocallyNoetherian_iff_of_iSup_eq_top {X : AlgebraicGeometry.Scheme} {ι : Sort u_1} {S : ιX.affineOpens} (hS : ⨆ (i : ι), (S i) = ) :
    AlgebraicGeometry.IsLocallyNoetherian X ∀ (i : ι), IsNoetherianRing (X.presheaf.obj (Opposite.op (S i)))

    A scheme is locally Noetherian if and only if it is covered by affine opens whose sections are noetherian rings.

    See [Har77], Proposition II.3.2.

    theorem AlgebraicGeometry.isLocallyNoetherian_iff_of_affine_openCover {X : AlgebraicGeometry.Scheme} (𝒰 : X.OpenCover) [∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)] :
    AlgebraicGeometry.IsLocallyNoetherian X ∀ (i : 𝒰.J), IsNoetherianRing ((𝒰.obj i).presheaf.obj (Opposite.op ))

    A version of isLocallyNoetherian_iff_of_iSup_eq_top using Scheme.OpenCover.

    If 𝒰 is an open cover of a scheme X, then X is locally noetherian if and only if 𝒰.obj i are all locally noetherian.

    If R is a noetherian ring, Spec R is a noetherian topological space.

    Equations
    • =
    @[instance 100]

    A locally Noetherian scheme is quasi-separated.

    Stacks: Lemma 01OY

    Equations
    • =

    A scheme X is Noetherian if it is locally Noetherian and compact.

      Instances
        theorem AlgebraicGeometry.isNoetherian_iff_of_finite_iSup_eq_top {X : AlgebraicGeometry.Scheme} {ι : Sort u_1} [Finite ι] {S : ιX.affineOpens} (hS : ⨆ (i : ι), (S i) = ) :
        AlgebraicGeometry.IsNoetherian X ∀ (i : ι), IsNoetherianRing (X.presheaf.obj (Opposite.op (S i)))

        A scheme is Noetherian if and only if it is covered by finitely many affine opens whose sections are noetherian rings.

        theorem AlgebraicGeometry.isNoetherian_iff_of_finite_affine_openCover {X : AlgebraicGeometry.Scheme} {𝒰 : X.OpenCover} [Finite 𝒰.J] [∀ (i : 𝒰.J), AlgebraicGeometry.IsAffine (𝒰.obj i)] :
        AlgebraicGeometry.IsNoetherian X ∀ (i : 𝒰.J), IsNoetherianRing ((𝒰.obj i).presheaf.obj (Opposite.op ))

        A version of isNoetherian_iff_of_finite_iSup_eq_top using Scheme.OpenCover.

        @[instance 100]

        A Noetherian scheme has a Noetherian underlying topological space.

        Stacks, Lemma 01OZ

        Equations
        • =
        @[instance 100]

        Any morphism of schemes f : X ⟶ Y with X Noetherian is quasi-compact.

        Stacks, Lemma 01P0

        Equations
        • =

        If R is a Noetherian ring, Spec R is a locally Noetherian scheme.

        Equations
        • =

        If R is a Noetherian ring, Spec R is a Noetherian scheme.

        Equations
        • =

        R is a Noetherian ring if and only if Spec R is a Noetherian scheme.

        A Noetherian scheme has a finite number of irreducible components.

        Stacks, Lemma 0BA8