Quadratic forms over the complex numbers #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
equivalent_sum_squares
: A nondegenerate quadratic form over the complex numbers is equivalent to
a sum of squares.
The isometry between a weighted sum of squares on the complex numbers and the
sum of squares, i.e. weighted_sum_squares
with weights 1 or 0.
Equations
- quadratic_form.isometry_sum_squares w' = let w : ι → ℂˣ := λ (i : ι), dite (w' i = 0) (λ (h : w' i = 0), 1) (λ (h : ¬w' i = 0), units.mk0 (w' i) h) in _.mpr ((quadratic_form.weighted_sum_squares ℂ w').isometry_basis_repr ((pi.basis_fun ℂ ι).units_smul (λ (i : ι), _.unit)))
The isometry between a weighted sum of squares on the complex numbers and the
sum of squares, i.e. weighted_sum_squares
with weight λ i : ι, 1
.
Equations
A nondegenerate quadratic form on the complex numbers is equivalent to
the sum of squares, i.e. weighted_sum_squares
with weight λ i : ι, 1
.
All nondegenerate quadratic forms on the complex numbers are equivalent.