Documentation

Mathlib.LinearAlgebra.CliffordAlgebra.Even

The universal property of the even subalgebra #

Main definitions #

Implementation notes #

The approach here is outlined in "Computing with the universal properties of the Clifford algebra and the even subalgebra" (to appear).

The broad summary is that we have two tricks available to us for implementing complex recursors on top of CliffordAlgebra.lift: the first is to use morphisms as the output type, such as A = Module.End R N which is how we obtained CliffordAlgebra.foldr; and the second is to use N = (N', S) where N' is the value we wish to compute, and S is some auxiliary state passed between one recursor invocation and the next. For the universal property of the even subalgebra, we apply a variant of the first trick again by choosing S to itself be a submodule of morphisms.

The even submodule CliffordAlgebra.evenOdd Q 0 is also a subalgebra.

Equations
Instances For
    @[simp]
    theorem CliffordAlgebra.even_toSubmodule {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] (Q : QuadraticForm R M) :
    Subalgebra.toSubmodule (CliffordAlgebra.even Q) = CliffordAlgebra.evenOdd Q 0
    theorem CliffordAlgebra.EvenHom.ext {R : Type uR} {M : Type uM} :
    ∀ {inst : CommRing R} {inst_1 : AddCommGroup M} {inst_2 : Module R M} {Q : QuadraticForm R M} {A : Type uA} {inst_3 : Ring A} {inst_4 : Algebra R A} (x y : CliffordAlgebra.EvenHom Q A), x.bilin = y.bilinx = y
    theorem CliffordAlgebra.EvenHom.ext_iff {R : Type uR} {M : Type uM} :
    ∀ {inst : CommRing R} {inst_1 : AddCommGroup M} {inst_2 : Module R M} {Q : QuadraticForm R M} {A : Type uA} {inst_3 : Ring A} {inst_4 : Algebra R A} (x y : CliffordAlgebra.EvenHom Q A), x = y x.bilin = y.bilin
    structure CliffordAlgebra.EvenHom {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] (Q : QuadraticForm R M) (A : Type uA) [Ring A] [Algebra R A] :
    Type (max uA uM)

    The type of bilinear maps which are accepted by CliffordAlgebra.even.lift.

    • bilin : M →ₗ[R] M →ₗ[R] A
    • contract : ∀ (m : M), (self.bilin m) m = (algebraMap R A) (Q m)
    • contract_mid : ∀ (m₁ m₂ m₃ : M), (self.bilin m₁) m₂ * (self.bilin m₂) m₃ = Q m₂ (self.bilin m₁) m₃
    Instances For
      @[simp]
      theorem CliffordAlgebra.EvenHom.compr₂_bilin {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} {B : Type uB} [Ring A] [Ring B] [Algebra R A] [Algebra R B] (g : CliffordAlgebra.EvenHom Q A) (f : A →ₐ[R] B) :
      def CliffordAlgebra.EvenHom.compr₂ {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} {B : Type uB} [Ring A] [Ring B] [Algebra R A] [Algebra R B] (g : CliffordAlgebra.EvenHom Q A) (f : A →ₐ[R] B) :

      Compose an EvenHom with an AlgHom on the output.

      Equations
      Instances For

        The embedding of pairs of vectors into the even subalgebra, as a bilinear map.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          Two algebra morphisms from the even subalgebra are equal if they agree on pairs of generators.

          See note [partially-applied ext lemmas].

          def CliffordAlgebra.even.lift.aux {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} [Ring A] [Algebra R A] (f : CliffordAlgebra.EvenHom Q A) :

          The final auxiliary construction for CliffordAlgebra.even.lift. This map is the forwards direction of that equivalence, but not in the fully-bundled form.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem CliffordAlgebra.even.lift.aux_one {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} [Ring A] [Algebra R A] (f : CliffordAlgebra.EvenHom Q A) :
            @[simp]
            theorem CliffordAlgebra.even.lift.aux_ι {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} [Ring A] [Algebra R A] (f : CliffordAlgebra.EvenHom Q A) (m₁ : M) (m₂ : M) :
            (CliffordAlgebra.even.lift.aux f) (((CliffordAlgebra.even.ι Q).bilin m₁) m₂) = (f.bilin m₁) m₂
            @[simp]
            theorem CliffordAlgebra.even.lift.aux_algebraMap {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] {Q : QuadraticForm R M} {A : Type uA} [Ring A] [Algebra R A] (f : CliffordAlgebra.EvenHom Q A) (r : R) (hr : (algebraMap R (CliffordAlgebra Q)) r CliffordAlgebra.even Q) :
            (CliffordAlgebra.even.lift.aux f) { val := (algebraMap R (CliffordAlgebra Q)) r, property := hr } = (algebraMap R A) r
            def CliffordAlgebra.even.lift {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] (Q : QuadraticForm R M) {A : Type uA} [Ring A] [Algebra R A] :

            Every algebra morphism from the even subalgebra is in one-to-one correspondence with a bilinear map that sends duplicate arguments to the quadratic form, and contracts across multiplication.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              theorem CliffordAlgebra.even.lift_ι {R : Type uR} {M : Type uM} [CommRing R] [AddCommGroup M] [Module R M] (Q : QuadraticForm R M) {A : Type uA} [Ring A] [Algebra R A] (f : CliffordAlgebra.EvenHom Q A) (m₁ : M) (m₂ : M) :
              ((CliffordAlgebra.even.lift Q) f) (((CliffordAlgebra.even.ι Q).bilin m₁) m₂) = (f.bilin m₁) m₂