mathlib3 documentation

lean-ga / geometric_algebra.from_mathlib.zmod_grading

Grading by ℤ / 2ℤ #

This file defines the grading by zmod 2, as the function clifford_algebra.grades'.

Main results #

Separate an element of the clifford algebra into its zmod 2-graded components.

This is defined as an alg_hom to add_monoid_algebra so that algebra operators can be moved before and after the mapping.

This is not the normal ℕ-graded definition that we usually use in GA. That definition is harder...

Equations

Recombining the grades recovers the original element

Stated another way, grades' has a left-inverse and is therefore injective (via function.left_inverse.injective).

@[protected, instance]
noncomputable def clifford_algebra.has_coe {R : Type u_1} [comm_ring R] {M : Type u_2} [add_comm_group M] [module R M] {Q : quadratic_form R M} :
Equations
@[simp, norm_cast]

An element of R lifted with algebra_map has a single grade 0 element

An element of X lifted with the canonical ι R function has a single grade 1 element