Commit 2024-02-16 17:31 29c27c39
View on Github →feat(LinearAlgebra/{ExteriorAlgebra,CliffordAlgebra}): Functoriality of the exterior algebra and some lemmas about generation (#9718) This does a few things:
- Define the algebra morphism
TrivSqZeroExt.map fbetween trivial square-zero extensions induced by a linear mapf, and establish some of its basic properties (functoriality, composition with the basic maps to/fromTrivSqZeroExt). Note that we only consider the case of a commutative base ring, because the case of a general base ring requires morphisms of bimodules, which we do not have. - Define the algebra morphism
ExteriorAlgebra.map fbetween exterior algebras induced by a linear mapf. This is a straightforward application of the similar construction for Clifford algebras, but I think it is still useful to have. Basic properties of this construction are proved: functoriality, composition withExteriorAlgebra.ι,ExteriorAlgebra.ιInv(this part uses the first point) andExteriorAlgebra.ιMulti. Then exactness properties of the construction is studied:- If the linear map is surjective, then the map on exterior algebras is also surjective. This actually holds for Clifford algebras, so I added a lemma called
CliffordAlgebra.map_surjectiveinLinearAlgebra/CliffordAlgebra/Basic.lean. For exterior algebras, the converse holds and is also proved. - If the linear map has a retraction, then the map on exterior algebras is injective. So if the base ring is a field, the map on exterior algebras is injective if the linear map is injective.
- If the linear map is surjective, then the map on exterior algebras is also surjective. This actually holds for Clifford algebras, so I added a lemma called
- Establish some properties of
ExteriorAlgebra.ιMulti:ExteriorAlgebra.ιMulti_range: The range ofιMulti R nis contained in thenth exterior power (define here asLinearMap.range (ι R : M →ₗ[R] ExteriorAlgebra R M) ^ n).ExteriorAlgebra.ιMulti_span_fixedDegree: This range spans thenth exterior power.ExteriorAlgebra.ιMulti_span: The union over allnof the range ofιMulti R nspans the whole exterior algebra (this is inLinearAlgebra/ExteriorAlgebra/Grading.leanbecause the proof uses the graded module structure, but it might be possible to do something simpler).
- Construct
ExteriorAlgebra.ιMulti_family: This takes a natural numbernand a family of vectorsvindexed by a linearly ordered typeI, and it returns the family ofn-fold products of thev iin the exterior algebra, indexed by the set of finsets ofIof cardinalityn. (The point, to be proved in another PR, is that whenvis a basis, thenExteriorAlgebra.ιMulti_family R n vis a basis of thenth exterior power.)