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
- SubmersivePresentation.free_cotangent:- I ⧸ I ^ 2is- S-free on the classes of- P.relation i.
- SubmersivePresentation.subsingleton_h1Cotangent:- H¹(L_{S/R}) = 0.
- SubmersivePresentation.free_kaehlerDifferential:- Ω[S⁄R]is- S-free on the images of- dxᵢwhere- i ∉ Set.range P.map.
- SubmersivePresentation.rank_kaehlerDifferential: If- Sis non-trivial, the rank of- Ω[S⁄R]is the dimension of- P.
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 : σ induced by the injection P.map : σ → ι.
If P is submersive, this is an isomorphism. See SubmersivePresentation.cotangentEquiv.
Equations
Instances For
The isomorphism of S-modules between I ⧸ I ^ 2 and σ → S given
by P.relation i ↦ ∂ⱼ (P.relation i).
Equations
Instances For
If P is a submersive presentation, H¹ of the associated cotangent complex vanishes.
The classes of P.relation i form a basis of I ⧸ I ^ 2.
Equations
Instances For
Stacks Tag 00T7 ((3))
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 σ and composing with the
inverse of P.cotangentEquiv.
By SubmersivePresentation.sectionCotangent_comp this is indeed a section.
Equations
- P.sectionCotangent = ↑P.cotangentEquiv.symm ∘ₗ ↑(Finsupp.linearEquivFunOnFinite S S σ) ∘ₗ Finsupp.lcomapDomain P.map ⋯ ∘ₗ ↑P.cotangentSpaceBasis.repr
Instances For
Alias of Algebra.SubmersivePresentation.sectionCotangent_zero_of_notMem_range.
Given a submersive presentation of S as R-algebra, any indexing type κ complementary to
the σ in ι indexes a basis of Ω[S⁄R].
See SubmersivePresentation.basisKaehler for the special case κ = (Set.range P.map)ᶜ.
Equations
- P.basisKaehlerOfIsCompl hf hcompl = Module.Basis.ofSplitExact ⋯ ⋯ ⋯ P.cotangentSpaceBasis hf ⋯ ⋯ ⋯
Instances For
Given a submersive presentation of S as R-algebra, the images of dxᵢ
for i in the complement of σ in ι form a basis of Ω[S⁄R].
Equations
- P.basisKaehler = P.basisKaehlerOfIsCompl ⋯ ⋯
Instances For
If P is a submersive presentation of S as an R-algebra, Ω[S⁄R] is free.
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.
The image of g * X - 1 in I/I² if I is the kernel of the canonical presentation
of the localization of S away from g.
Equations
Instances For
The basis of (g * X - 1) / (g * X - 1)² given by the image of g * X - 1.
This is def-eq to (SubmersivePresentation.localizationAway T g).basisCotangent, but
(SubmersivePresentation.localizationAway T g).toExtension =
  (Generators.localizationAway T g).toExtension
is not reducibly def-eq. Hence using the general SubmersivePresentation.basisCotangent leads
to erw hell.
Equations
Instances For
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.
If S is R-standard smooth of relative dimension zero, it is étale.