mathlib3 documentation

lean-ga / geometric_algebra.from_mathlib.conjugation

Conjugations #

This file contains additional lemmas about clifford_algebra.reverse and clifford_algebra.involute.

As more and more goes into Mathlib, this file will become smaller and spaller. The links above will take you to the collection of mathlib theorems.

theorem clifford_algebra.reverse_prod_sign_aux {R : Type u_1} [comm_ring R] (n : ) :
(-1) ^ ((n + 1) * (n + 1 + 1) / 2) = (-1) ^ (n * (n + 1) / 2) * (-1) ^ (n + 1)

helper lemma for expanding the sign of reverse

TODO: this needs an assumption that the vectors are othogonal

Note: this declaration is incomplete and uses sorry.