Documentation

Mathlib.AlgebraicGeometry.IdealSheaf

Ideal sheaves on schemes #

We define ideal sheaves of schemes and provide various constructors for it.

Main definition #

Main results #

Implementation detail #

Ideal sheaves are not yet defined in this file as actual subsheaves of 𝒪ₓ. Instead, for the ease of development and application, we define the structure IdealSheafData containing all necessary data to uniquely define an ideal sheaf. This should be refectored as a constructor for ideal sheaves once they are introduced into mathlib.

A structure that contains the data to uniquely define an ideal sheaf, consisting of

  1. an ideal I(U) ≤ Γ(X, U) for every affine open U
  2. a proof that I(D(f)) = I(U)_f for every affine open U and every section f : Γ(X, U).
Instances For

    The largest ideal sheaf contained in a family of ideals.

    Equations
    Instances For

      The galois coinsertion between ideal sheaves and arbitrary families of ideals.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem AlgebraicGeometry.Scheme.IdealSheafData.ideal_iSup {X : Scheme} {ι : Type u_1} {I : ιX.IdealSheafData} :
        (iSup I).ideal = ⨆ (i : ι), (I i).ideal
        @[simp]
        theorem AlgebraicGeometry.Scheme.IdealSheafData.ideal_biInf {X : Scheme} {ι : Type u_1} (I : ιX.IdealSheafData) {s : Set ι} (hs : s.Finite) :
        (⨅ is, I i).ideal = is, (I i).ideal
        @[simp]
        theorem AlgebraicGeometry.Scheme.IdealSheafData.ideal_iInf {X : Scheme} {ι : Type u_1} (I : ιX.IdealSheafData) [Finite ι] :
        (⨅ (i : ι), I i).ideal = ⨅ (i : ι), (I i).ideal

        A form of map_ideal that is easier to rewrite with.

        The ideal sheaf induced by an ideal of the global sections.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem AlgebraicGeometry.Scheme.IdealSheafData.le_of_isAffine {X : Scheme} [IsAffine X] {I J : X.IdealSheafData} (H : I.ideal , J.ideal , ) :
          I J
          theorem AlgebraicGeometry.Scheme.IdealSheafData.ext_of_isAffine {X : Scheme} [IsAffine X] {I J : X.IdealSheafData} (H : I.ideal , = J.ideal , ) :
          I = J

          Over affine schemes, ideal sheaves are in bijection with ideals of the global sections.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            The support of an ideal sheaf. Also see IdealSheafData.mem_support_iff_of_mem.

            Equations
            Instances For

              The radical of a ideal sheaf.

              Equations
              Instances For

                The nilradical of a scheme.

                Equations
                Instances For

                  The vanishing ideal sheaf of a set, which is the largest ideal sheaf whose support contains a subset. When the set Z is closed, the reduced induced scheme structure is the quotient of this ideal.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    support and vanishingIdeal forms a galois connection. This is the global version of PrimeSpectrum.gc.

                    The kernel of a morphism, defined as the largest (quasi-coherent) ideal sheaf contained in the component-wise kernel. This is usually only well-behaved when f is quasi-compact.

                    Equations
                    Instances For
                      theorem AlgebraicGeometry.Scheme.ker_morphismRestrict_ideal {X Y : Scheme} (f : X.Hom Y) [QuasiCompact f] (U : Y.Opens) (V : (↑U).affineOpens) :
                      (Hom.ker (f ∣_ U)).ideal V = f.ker.ideal (Hom.opensFunctor U.ι).obj V,
                      theorem AlgebraicGeometry.Scheme.ker_ideal_of_isPullback_of_isOpenImmersion {X Y U V : Scheme} (f : X Y) (f' : U V) (iU : U X) (iV : V Y) [IsOpenImmersion iV] [QuasiCompact f] (H : CategoryTheory.IsPullback f' iU iV f) (W : V.affineOpens) :

                      Spec (𝒪ₓ(U)/I(U)), the object to be glued into the closed subscheme.

                      Equations
                      Instances For

                        Spec (𝒪ₓ(U)/I(U)) ⟶ Spec (𝒪ₓ(U)) = U, the closed immersion into U.

                        Equations
                        Instances For

                          The open immersion Spec Γ(𝒪ₓ/I, U) ⟶ Spec Γ(𝒪ₓ/I, V) if U ≤ V.

                          Equations
                          Instances For
                            @[reducible, inline]

                            The intersections Spec Γ(𝒪ₓ/I, U) ∩ V useful for gluing.

                            Equations
                            Instances For

                              (Implementation) Transition maps in the glue data for 𝒪ₓ/I.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For

                                (Implementation) t' in the glue data for 𝒪ₓ/I.

                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For

                                  (Implementation) The glue data for 𝒪ₓ/I.

                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    @[simp]
                                    theorem AlgebraicGeometry.Scheme.IdealSheafData.glueData_t' {X : Scheme} (I : X.IdealSheafData) (i j k : X.affineOpens) :
                                    I.glueData.t' i j k = CategoryTheory.Limits.pullback.lift (I.glueDataT'Aux (i, j).1 (i, j).2 (i, k).2 (j, k).2 ) (I.glueDataT'Aux (i, j).1 (i, j).2 (i, k).2 (j, i).2 )