Bilinear form #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the conversion between bilinear forms and matrices.
Main definitions #
matrix.to_bilin
given a basis define a bilinear formmatrix.to_bilin'
define the bilinear form onn → R
bilin_form.to_matrix
: calculate the matrix coefficients of a bilinear formbilin_form.to_matrix'
: calculate the matrix coefficients of a bilinear form onn → R
Notations #
In this file we use the following type variables:
M
,M'
, ... are modules over the semiringR
,M₁
,M₁'
, ... are modules over the ringR₁
,M₂
,M₂'
, ... are modules over the commutative semiringR₂
,M₃
,M₃'
, ... are modules over the commutative ringR₃
,V
, ... is a vector space over the fieldK
.
Tags #
bilinear_form, matrix, basis
The map from matrix n n R
to bilinear forms on n → R
.
This is an auxiliary definition for the equivalence matrix.to_bilin_form'
.
Equations
- M.to_bilin'_aux = {bilin := λ (v w : n → R₂), finset.univ.sum (λ (i : n), finset.univ.sum (λ (j : n), v i * M i j * w j)), bilin_add_left := _, bilin_smul_left := _, bilin_add_right := _, bilin_smul_right := _}
The linear map from bilinear forms to matrix n n R
given an n
-indexed basis.
This is an auxiliary definition for the equivalence matrix.to_bilin_form'
.
Equations
- bilin_form.to_matrix_aux b = {to_fun := λ (B : bilin_form R₂ M₂), ⇑matrix.of (λ (i j : n), ⇑B (b i) (b j)), map_add' := _, map_smul' := _}
to_matrix'
section #
This section deals with the conversion between matrices and bilinear forms on n → R₂
.
The linear equivalence between bilinear forms on n → R
and n × n
matrices
Equations
- bilin_form.to_matrix' = {to_fun := (bilin_form.to_matrix_aux (λ (j : n), ⇑(linear_map.std_basis R₂ (λ (_x : n), R₂) j) 1)).to_fun, map_add' := _, map_smul' := _, inv_fun := matrix.to_bilin'_aux _inst_16, left_inv := _, right_inv := _}
The linear equivalence between n × n
matrices and bilinear forms on n → R
Equations
to_matrix
section #
This section deals with the conversion between matrices and bilinear forms on a module with a fixed basis.
bilin_form.to_matrix b
is the equivalence between R
-bilinear forms on M
and
n
-by-n
matrices with entries in R
, if b
is an R
-basis for M
.
Equations
bilin_form.to_matrix b
is the equivalence between R
-bilinear forms on M
and
n
-by-n
matrices with entries in R
, if b
is an R
-basis for M
.
Equations
The submodule of pair-self-adjoint matrices with respect to bilinear forms corresponding to
given matrices J
, J₂
.
The submodule of self-adjoint matrices with respect to the bilinear form corresponding to
the matrix J
.
Equations
The submodule of skew-adjoint matrices with respect to the bilinear form corresponding to
the matrix J
.