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 ^ 2
isS
-free on the classes ofP.relation i
.SubmersivePresentation.subsingleton_h1Cotangent
:H¹(L_{S/R}) = 0
.SubmersivePresentation.free_kaehlerDifferential
:Ω[S⁄R]
isS
-free on the images ofdxᵢ
wherei ∉ Set.range P.map
.SubmersivePresentation.rank_kaehlerDifferential
: IfS
is non-trivial, the rank ofΩ[S⁄R]
is the dimension ofP
.
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
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
.
Stacks Tag 00T7 ((3))
Equations
- P.basisCotangent = { repr := P.cotangentEquiv.trans (Finsupp.linearEquivFunOnFinite S S P.rels).symm }
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 P.rels
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 P.rels) ∘ₗ Finsupp.lcomapDomain P.map ⋯ ∘ₗ ↑P.cotangentSpaceBasis.repr
Instances For
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
- P.basisKaehlerOfIsCompl hf hcompl = 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 P.rels
in P.vars
form a basis of Ω[S⁄R]
.
Stacks Tag 00T7 ((2))
Equations
- P.basisKaehler = P.basisKaehlerOfIsCompl ⋯ ⋯
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
.
If S
is R
-standard smooth of relative dimension zero, it is étale.