Exterior powers #
We study the exterior powers of a module M
over a commutative ring R
.
Definitions #
exteriorPower.ιMulti
is the canonical alternating map onM
with values in⋀[R]^n M
.exteriorPower.presentation R n M
is the standard presentation of theR
-module⋀[R]^n M
.
Theorems #
ιMulti_span
: The image ofexteriorPower.ιMulti
spans⋀[R]^n M
.We construct
exteriorPower.alternatingMapLinearEquiv
which expresses the universal property of the exterior power as a linear equivalence(M [⋀^Fin n]→ₗ[R] N) ≃ₗ[R] ⋀[R]^n M →ₗ[R] N
between alternating maps and linear maps from the exterior power.
The canonical alternating map from Fin n → M
to ⋀[R]^n M
.
exteriorAlgebra.ιMulti
is the alternating map from Fin n → M
to ⋀[r]^n M
induced by exteriorAlgebra.ιMulti
, i.e. sending a family of vectors m : Fin n → M
to the
product of its entries.
Equations
- exteriorPower.ιMulti R n = (ExteriorAlgebra.ιMulti R n).codRestrict (⋀[R]^n M) ⋯
Instances For
The image of ExteriorAlgebra.ιMulti R n
spans the n
th exterior power. Variant of
ExteriorAlgebra.ιMulti_span_fixedDegree
, useful in rewrites.
The image of exteriorPower.ιMulti
spans ⋀[R]^n M
.
The index type for the relations in the standard presentation of ⋀[R]^n M
,
in the particular case ι
is Fin n
.
- add {R : Type u} {ι : Type u_4} {M : Type u_5} (m : ι → M) (i : ι) (x y : M) : exteriorPower.presentation.Rels R ι M
- smul {R : Type u} {ι : Type u_4} {M : Type u_5} (m : ι → M) (i : ι) (r : R) (x : M) : exteriorPower.presentation.Rels R ι M
- alt {R : Type u} {ι : Type u_4} {M : Type u_5} (m : ι → M) (i j : ι) (hm : m i = m j) (hij : i ≠ j) : exteriorPower.presentation.Rels R ι M
Instances For
The relations in the standard presentation of ⋀[R]^n M
with generators and relations.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The solutions in a module N
to the linear equations
given by exteriorPower.relations R ι M
identify to alternating maps to N
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The universal property of the exterior power.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The standard presentation of the R
-module ⋀[R]^n M
.
Equations
Instances For
Two linear maps on ⋀[R]^n M
that agree on the image of exteriorPower.ιMulti
are equal.
The linear equivalence between n
-fold alternating maps from M
to N
and linear maps from
⋀[R]^n M
to N
: this is the universal property of the n
th exterior power of M
.
Equations
- exteriorPower.alternatingMapLinearEquiv = ((⋯.linearMapEquiv.trans exteriorPower.presentation.relationsSolutionEquiv).toLinearEquiv ⋯).symm
Instances For
If f
is an alternating map from M
to N
,
alternatingMapLinearEquiv f
is the corresponding linear map from ⋀[R]^n M
to N
,
and if g
is a linear map from N
to N'
, then
the alternating map g.compAlternatingMap f
from M
to N'
corresponds to the linear
map g.comp (alternatingMapLinearEquiv f)
on ⋀[R]^n M
.