mathlib3 documentation

lean-ga / geometric_algebra.from_mathlib.basic

@[reducible]
def clifford_algebra.clifford_hom {R : Type u_1} [comm_ring R] {M : Type u_2} [add_comm_group M] [module R M] (Q : quadratic_form R M) (A : Type u_3) [semiring A] [algebra R A] :
Type (max u_2 u_3)
theorem clifford_algebra.preserves_iff_bilin {R : Type u_1} [comm_ring R] {M : Type u_2} [add_comm_group M] [module R M] (Q : quadratic_form R M) {A : Type u_3} [ring A] [algebra R A] (h2 : is_unit 2) (f : M →ₗ[R] A) :

A wedge product of n vectors. Note this does not define the wedge product of arbitrary multivectors.

Equations