Complexification of a clifford algebra #
In this file we show the isomorphism
clifford_algebra.equiv_complexify Q : clifford_algebra Q.complexify ≃ₐ[ℂ] (ℂ ⊗[ℝ] clifford_algebra Q)
with forward directionclifford_algebra.to_complexify Q
and reverse directionclifford_algebra.of_complexify Q
.
where
quadratic_form.complexify Q : quadratic_form ℂ (ℂ ⊗[ℝ] V)
, which is defined in terms of a more generalquadratic_form.base_change
.
This covers §2.2 of https://empg.maths.ed.ac.uk/Activities/Spin/Lecture2.pdf.
We show:
clifford_algebra.to_complexify_ι
: the effect of complexifying pure vectors.clifford_algebra.of_complexify_tmul_ι
: the effect of un-complexifying a tensor of pure vectors.clifford_algebra.to_complexify_involute
: the effect of complexifying an involution.clifford_algebra.to_complexify_reverse
: the effect of complexifying a reversal.
Note that all the results in this file are already in Mathlib4 due to https://github.com/leanprover-community/mathlib4/pull/6778.
Change the base of a quadratic form, defined by $Q_A(a ⊗_R v) = a^2Q(v)$.
Equations
The complexification of a quadratic form, defined by $Q_ℂ(z ⊗ v) = z^2Q(v)$.
Equations
Equations
Equations
Equations
Auxiliary construction: note this is really just a heterobasic clifford_algebra.map
.
Equations
Convert from the complexified clifford algebra to the clifford algebra over a complexified module.
Equations
- clifford_algebra.of_complexify Q = algebra.tensor_product.alg_hom_of_linear_map_tensor_product' (tensor_product.algebra_tensor_module.lift (let f : ℂ →ₗ[ℂ] module.End ℂ (clifford_algebra Q.complexify) := (algebra.lsmul ℂ (clifford_algebra Q.complexify)).to_linear_map in (({to_fun := λ (f : clifford_algebra Q.complexify →ₗ[ℂ] clifford_algebra Q.complexify), linear_map.restrict_scalars ℝ f, map_add' := _, map_smul' := _}.comp f).flip.comp (clifford_algebra.of_complexify_aux Q).to_linear_map).flip)) _ _
Convert from the clifford algebra over a complexified module to the complexified clifford algebra.
Equations
- clifford_algebra.to_complexify Q = ⇑(clifford_algebra.lift Q.complexify) (let φ : tensor_product ℝ ℂ V →ₗ[ℂ] tensor_product ℝ ℂ (clifford_algebra Q) := tensor_product.algebra_tensor_module.map linear_map.id (clifford_algebra.ι Q) in ⟨φ, _⟩)
The involution acts only on the right of the tensor product.
Auxiliary lemma used to prove to_complexify_reverse
without needing induction.
reverse
acts only on the right of the tensor product.
Complexifying the vector space of a clifford algebra is isomorphic as a ℂ-algebra to complexifying the clifford algebra itself; $Cℓ(ℂ ⊗_ℝ V, Q_ℂ) ≅ ℂ ⊗_ℝ Cℓ(V, Q)$.
This is clifford_algebra.to_complexify
and clifford_algebra.of_complexify
as an equivalence.