Isometric equivalences with respect to quadratic forms #
Main definitions #
QuadraticForm.IsometryEquiv
:LinearEquiv
s which map between two different quadratic formsQuadraticForm.Equivalent
: propositional version of the above
Main results #
equivalent_weighted_sum_squares
: in finite dimensions, any quadratic form is equivalent to a parametrization ofQuadraticForm.weightedSumSquares
.
- toFun : M₁ → M₂
- map_add' : ∀ (x y : M₁), AddHom.toFun s.toAddHom (x + y) = AddHom.toFun s.toAddHom x + AddHom.toFun s.toAddHom y
- map_smul' : ∀ (r : R) (x : M₁), AddHom.toFun s.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun s.toAddHom x
- invFun : M₂ → M₁
- left_inv : Function.LeftInverse s.invFun s.toFun
- right_inv : Function.RightInverse s.invFun s.toFun
- map_app' : ∀ (m : M₁), ↑Q₂ (AddHom.toFun s.toAddHom m) = ↑Q₁ m
An isometric equivalence between two quadratic spaces M₁, Q₁
and M₂, Q₂
over a ring R
,
is a linear equivalence between M₁
and M₂
that commutes with the quadratic forms.
Instances For
Two quadratic forms over a ring R
are equivalent
if there exists an isometric equivalence between them:
a linear equivalence that transforms one quadratic form into the other.
Instances For
The identity isometric equivalence between a quadratic form and itself.
Instances For
The inverse isometric equivalence of an isometric equivalence between two quadratic forms.
Instances For
The composition of two isometric equivalences between quadratic forms.
Instances For
Isometric equivalences are isometric maps
Instances For
A quadratic form composed with a LinearEquiv
is isometric to itself.
Instances For
A quadratic form is isometrically equivalent to its bases representations.
Instances For
Given an orthogonal basis, a quadratic form is isometrically equivalent with a weighted sum of squares.