Documentation

Mathlib.AlgebraicGeometry.Modules.Tilde

Construction of M^~ #

Given any commutative ring R and R-module M, we construct the sheaf M^~ of 𝒪_SpecR-modules such that M^~(U) is the set of dependent functions that are locally fractions.

Main definitions #

@[reducible, inline]

For an R-module M and a point P in Spec R, Localizations P is the localized module M at the prime ideal P.

Equations
Instances For

    For any open subset U ⊆ Spec R, IsFraction is the predicate expressing that a function f : ∏_{x ∈ U}, Mₓ is such that for any 𝔭 ∈ U, f 𝔭 = m / s for some m : M and s ∉ 𝔭. In short f is a fraction on U.

    Equations
    Instances For

      The property of a function f : ∏_{x ∈ U}, Mₓ being a fraction is stable under restriction.

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

        For any open subset U ⊆ Spec R, IsLocallyFraction is the predicate expressing that a function f : ∏_{x ∈ U}, Mₓ is such that for any 𝔭 ∈ U, there exists an open neighbourhood V ∋ 𝔭, such that for any 𝔮 ∈ V, f 𝔮 = m / s for some m : M and s ∉ 𝔮. In short f is locally a fraction on U.

        Equations
        Instances For
          @[simp]
          theorem ModuleCat.Tilde.isLocallyFraction_pred {R : Type u} [CommRing R] (M : ModuleCat R) {U : TopologicalSpace.Opens (AlgebraicGeometry.PrimeSpectrum.Top R)} (f : (x : U) → ModuleCat.Tilde.Localizations M x) :
          (ModuleCat.Tilde.isLocallyFraction M).pred f = ∀ (y : U), ∃ (V : TopologicalSpace.Opens (AlgebraicGeometry.PrimeSpectrum.Top R)) (_ : y V) (i : V U) (m : M) (s : R), ∀ (x : V), s(x).asIdeal s f ((fun (x : V) => x, ) x) = (LocalizedModule.mkLinearMap (x).asIdeal.primeCompl M) m

          For any R-module M and any open subset U ⊆ Spec R, M^~(U) is an 𝒪_{Spec R}(U)-submodule of ∏_{𝔭 ∈ U} M_𝔭.

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

            For any R-module M, TildeInType R M is the sheaf of set on Spec R whose sections on U are the dependent functions that are locally fractions. This is often denoted by M^~.

            See also Tilde.isLocallyFraction.

            Equations
            Instances For
              Equations

              M^~ as a presheaf of abelian groups over Spec R

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

                M^~ as a sheaf of abelian groups over Spec R

                Equations
                • M.tildeInAddCommGrp = { val := M.preTildeInAddCommGrp, cond := }
                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  noncomputable def ModuleCat.tilde {R : Type u} [CommRing R] (M : ModuleCat R) :

                  M^~ as a sheaf of 𝒪_{Spec R}-modules

                  Equations
                  • M.tilde = { val := { presheaf := M.tildeInAddCommGrp.val, module := inferInstance, map_smul := }, isSheaf := }
                  Instances For