Sesquilinear form #
This files provides properties about sesquilinear forms. The maps considered are of the form
M₁ →ₛₗ[I₁] M₂ →ₛₗ[I₂] R
, where I₁ : R₁ →+* R
and I₂ : R₂ →+* R
are ring homomorphisms and
M₁
is a module over R₁
and M₂
is a module over R₂
.
Sesquilinear forms are the special case that M₁ = M₂
, R₁ = R₂ = R
, and I₁ = ring_hom.id R
.
Taking additionally I₂ = ring_hom.id R
, then one obtains bilinear forms.
These forms are a special case of the bilinear maps defined in bilinear_map.lean
and all basic
lemmas about construction and elementary calculations are found there.
Main declarations #
is_ortho
: states that two vectors are orthogonal with respect to a sesquilinear formis_symm
,is_alt
: states that a sesquilinear form is symmetric and alternating, respectivelyorthogonal_bilin
: provides the orthogonal complement with respect to sesquilinear form
References #
Tags #
Sesquilinear form,
Orthogonal vectors #
The proposition that two elements of a sesquilinear form space are orthogonal
A set of vectors v
is orthogonal with respect to some bilinear form B
if and only
if for all i ≠ j
, B (v i) (v j) = 0
. For orthogonality between two elements, use
bilin_form.is_ortho
A set of orthogonal vectors v
with respect to some sesquilinear form B
is linearly
independent if for all i
, B (v i) (v i) ≠ 0
.
Reflexive bilinear forms #
The proposition that a sesquilinear form is reflexive
Symmetric bilinear forms #
Alternating bilinear forms #
The orthogonal complement #
The orthogonal complement of a submodule N
with respect to some bilinear form is the set of
elements x
which are orthogonal to all elements of N
; i.e., for all y
in N
, B x y = 0
.
Note that for general (neither symmetric nor antisymmetric) bilinear forms this definition has a
chirality; in addition to this "left" orthogonal complement one could define a "right" orthogonal
complement for which, for all y
in N
, B y x = 0
. This variant definition is not currently
provided in mathlib.
Given a bilinear form B
and some x
such that B x x ≠ 0
, the span of the singleton of x
is complement to its orthogonal complement.