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 : 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 : Scheme} {ι : Sort u_1} {S : ι → ↑X.affineOpens} (hS : ⨆ (i : ι), ↑(S i) = ⊤) :
    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 : Scheme} (š’° : X.OpenCover) [āˆ€ (i : š’°.Iā‚€), IsAffine (š’°.X i)] :
    IsLocallyNoetherian X ↔ āˆ€ (i : š’°.Iā‚€), IsNoetherianRing ↑((š’°.X 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 š’°.X i are all locally Noetherian.

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

    @[instance 100]

    Any open immersion Z ⟶ X with X locally Noetherian is quasi-compact.

    @[instance 100]

    A locally Noetherian scheme is quasi-separated.

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

    Instances
      theorem AlgebraicGeometry.isNoetherian_iff_of_finite_iSup_eq_top {X : Scheme} {ι : Sort u_1} [Finite ι] {S : ι → ↑X.affineOpens} (hS : ⨆ (i : ι), ↑(S i) = ⊤) :
      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 : Scheme} {š’° : X.OpenCover} [Finite š’°.Iā‚€] [āˆ€ (i : š’°.Iā‚€), IsAffine (š’°.X i)] :
      IsNoetherian X ↔ āˆ€ (i : š’°.Iā‚€), IsNoetherianRing ↑((š’°.X 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.

      @[instance 100]

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

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

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

      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.