Real quadratic forms #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Sylvester's law of inertia equivalent_one_neg_one_weighted_sum_squared
:
A real quadratic form is equivalent to a weighted
sum of squares with the weights being ±1 or 0.
When the real quadratic form is nondegerate we can take the weights to be ±1,
as in equivalent_one_zero_neg_one_weighted_sum_squared
.
The isometry between a weighted sum of squares with weights u
on the
(non-zero) real numbers and the weighted sum of squares with weights sign ∘ u
.
Equations
- quadratic_form.isometry_sign_weighted_sum_squares w = let u : ι → ℝˣ := λ (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)))
Sylvester's law of inertia: A nondegenerate real quadratic form is equivalent to a weighted sum of squares with the weights being ±1.
Sylvester's law of inertia: A real quadratic form is equivalent to a weighted sum of squares with the weights being ±1 or 0.