Documentation

Mathlib.RingTheory.Smooth.StandardSmoothCotangent

Cotangent complex of a submersive presentation #

Let P be a submersive presentation of S as an R-algebra and denote by I the kernel R[X] → S. We show

We also provide the corresponding instances for standard smooth algebras as corollaries.

We keep the notation I = ker(R[X] → S) in all docstrings of this file.

Given a pre-submersive presentation, this is the composition I ⧸ I ^ 2 → ⊕ S dxᵢ → ⊕ S dxᵢ where the second direct sum runs over all i : P.rels induced by the injection P.map : P.rels → P.vars.

If P is submersive, this is an isomorphism. See SubmersivePresentation.cotangentEquiv.

Equations
Instances For

    The isomorphism of S-modules between I ⧸ I ^ 2 and P.rels → S given by P.relation i ↦ ∂ⱼ (P.relation i).

    Equations
    Instances For
      @[simp]
      theorem Algebra.SubmersivePresentation.cotangentEquiv_apply {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] (P : SubmersivePresentation R S) (a✝ : P.toExtension.Cotangent) (a✝¹ : P.rels) :
      P.cotangentEquiv a✝ a✝¹ = P.cotangentComplexAux a✝ a✝¹

      If P is a submersive presentation, of the associated cotangent complex vanishes.

      The classes of P.relation i form a basis of I ⧸ I ^ 2.

      Stacks Tag 00T7 ((3))

      Equations
      Instances For

        If P is a submersive presentation, this is the section of the map I ⧸ I ^ 2 → ⊕ S dxᵢ given by projecting to the summands indexed by P.rels and composing with the inverse of P.cotangentEquiv.

        By SubmersivePresentation.sectionCotangent_comp this is indeed a section.

        Equations
        Instances For
          noncomputable def Algebra.SubmersivePresentation.basisKaehlerOfIsCompl {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] (P : SubmersivePresentation R S) {κ : Type u_3} {f : κP.vars} (hf : Function.Injective f) (hcompl : IsCompl (Set.range f) (Set.range P.map)) :
          Basis κ S (Ω[SR])

          Given a submersive presentation of S as R-algebra, any indexing type κ complementary to the P.rels in P.vars indexes a basis of Ω[S⁄R]. See SubmersivePresentation.basisKaehler for the special case κ = (Set.range P.map)ᶜ.

          Equations
          Instances For
            noncomputable def Algebra.SubmersivePresentation.basisKaehler {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] (P : SubmersivePresentation R S) :
            Basis (↑(Set.range P.map)) S (Ω[SR])

            Given a submersive presentation of S as R-algebra, the images of dxᵢ for i in the complement of P.rels in P.vars form a basis of Ω[S⁄R].

            Stacks Tag 00T7 ((2))

            Equations
            Instances For

              If P is a submersive presentation of S as an R-algebra, Ω[S⁄R] is free.

              Stacks Tag 00T7 ((2))

              If P is a submersive presentation of S as an R-algebra and S is nontrivial, Ω[S⁄R] is free of rank the dimension of P, i.e. the number of generators minus the number of relations.

              If S is R-standard smooth, Ω[S⁄R] is a free S-module.

              If S is non-trivial and R-standard smooth of relative dimension, Ω[S⁄R] is a free S-module of rank n.

              @[instance 900]
              @[instance 900]

              If S is R-standard smooth of relative dimension zero, it is étale.