Exterior Algebras #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We construct the exterior algebra of a module M
over a commutative semiring R
.
Notation #
The exterior algebra of the R
-module M
is denoted as exterior_algebra R M
.
It is endowed with the structure of an R
-algebra.
Given a linear morphism f : M → A
from a module M
to another R
-algebra A
, such that
cond : ∀ m : M, f m * f m = 0
, there is a (unique) lift of f
to an R
-algebra morphism,
which is denoted exterior_algebra.lift R f cond
.
The canonical linear map M → exterior_algebra R M
is denoted exterior_algebra.ι R
.
Theorems #
The main theorems proved ensure that exterior_algebra R M
satisfies the universal property
of the exterior algebra.
ι_comp_lift
is fact that the composition ofι R
withlift R f cond
agrees withf
.lift_unique
ensures the uniqueness oflift R f cond
with respect to 1.
Definitions #
ι_multi
is thealternating_map
corresponding to the wedge product ofι R m
terms.
Implementation details #
The exterior algebra of M
is constructed as simply clifford_algebra (0 : quadratic_form R M)
,
as this avoids us having to duplicate API.
The exterior algebra of an R
-module M
.
Equations
The canonical linear map M →ₗ[R] exterior_algebra R M
.
Equations
As well as being linear, ι m
squares to zero
Given a linear map f : M →ₗ[R] A
into an R
-algebra A
, which satisfies the condition:
cond : ∀ m : M, f m * f m = 0
, this is the canonical lift of f
to a morphism of R
-algebras
from exterior_algebra R M
to A
.
Equations
- exterior_algebra.lift R = ((equiv.refl (M →ₗ[R] A)).subtype_equiv _).trans (clifford_algebra.lift 0)
If C
holds for the algebra_map
of r : R
into exterior_algebra R M
, the ι
of x : M
,
and is preserved under addition and muliplication, then it holds for all of exterior_algebra R M
.
The left-inverse of algebra_map
.
Equations
Invertibility in the exterior algebra is the same as invertibility of the base ring.
The canonical map from exterior_algebra R M
into triv_sq_zero_ext R M
that sends
exterior_algebra.ι
to triv_sq_zero_ext.inr
.
Equations
- exterior_algebra.to_triv_sq_zero_ext = ⇑(exterior_algebra.lift R) ⟨triv_sq_zero_ext.inr_hom R M _inst_3, _⟩
The left-inverse of ι
.
As an implementation detail, we implement this using triv_sq_zero_ext
which has a suitable
algebra structure.
Equations
- exterior_algebra.ι_inv = let _inst : module Rᵐᵒᵖ M := module.comp_hom M ((ring_hom.id R).from_opposite exterior_algebra.ι_inv._proof_1) in (triv_sq_zero_ext.snd_hom R M).comp exterior_algebra.to_triv_sq_zero_ext.to_linear_map
The generators of the exterior algebra are disjoint from its scalars.
The product of n
terms of the form ι R m
is an alternating map.
This is a special case of multilinear_map.mk_pi_algebra_fin
, and the exterior algebra version of
tensor_algebra.tprod
.
Equations
- exterior_algebra.ι_multi R n = let F : multilinear_map R (λ (i : fin n), M) (exterior_algebra R M) := (multilinear_map.mk_pi_algebra_fin R n (exterior_algebra R M)).comp_linear_map (λ (i : fin n), exterior_algebra.ι R) in {to_fun := ⇑F, map_add' := _, map_smul' := _, map_eq_zero_of_eq' := _}
The canonical image of the tensor_algebra
in the exterior_algebra
, which maps
tensor_algebra.ι R x
to exterior_algebra.ι R x
.