mathlib documentation

linear_algebra.sesquilinear_form

Sesquilinear form

This file defines a sesquilinear form over a module. The definition requires a ring antiautomorphism on the scalar ring. Basic ideas such as orthogonality are also introduced.

A sesquilinear form on an R-module M, is a function from M × M to R, that is linear in the first argument and antilinear in the second, with respect to an antiautomorphism on R (an antiisomorphism from R to R).

Notations

Given any term S of type sesq_form, due to a coercion, can use the notation S x y to refer to the function field, ie. S x y = S.sesq x y.

References

Tags

Sesquilinear form,

structure sesq_form (R : Type u) (M : Type v) [ring R] (I : R ≃+* Rᵒᵖ) [add_comm_group M] [module R M] :
Type (max u v)

A sesquilinear form over a module

@[instance]
def sesq_form.has_coe_to_fun {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} :

Equations
theorem sesq_form.add_left {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y z : M) :
S (x + y) z = S x z + S y z

theorem sesq_form.smul_left {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (a : R) (x y : M) :
S (a x) y = a * S x y

theorem sesq_form.add_right {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y z : M) :
S x (y + z) = S x y + S x z

theorem sesq_form.smul_right {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (a : R) (x y : M) :
S x (a y) = (opposite.unop (I a)) * S x y

theorem sesq_form.zero_left {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x : M) :
S 0 x = 0

theorem sesq_form.zero_right {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x : M) :
S x 0 = 0

theorem sesq_form.neg_left {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y : M) :
S (-x) y = -S x y

theorem sesq_form.neg_right {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y : M) :
S x (-y) = -S x y

theorem sesq_form.sub_left {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y z : M) :
S (x - y) z = S x z - S y z

theorem sesq_form.sub_right {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x y z : M) :
S x (y - z) = S x y - S x z

@[ext]
theorem sesq_form.ext {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S D : sesq_form R M I} (H : ∀ (x y : M), S x y = D x y) :
S = D

@[instance]
def sesq_form.add_comm_group {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} :

Equations
@[instance]
def sesq_form.inhabited {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} :

Equations
def sesq_form.is_ortho {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} (S : sesq_form R M I) (x y : M) :
Prop

The proposition that two elements of a sesquilinear form space are orthogonal

Equations
theorem sesq_form.ortho_zero {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (x : M) :
S.is_ortho 0 x

@[instance]
def sesq_form.to_module {R : Type u_1} [comm_ring R] {M : Type v} [add_comm_group M] [module R M] {J : R ≃+* Rᵒᵖ} :
module R (sesq_form R M J)

Equations
theorem sesq_form.ortho_smul_left {R : Type u_1} [domain R] {M : Type v} [add_comm_group M] [module R M] {K : R ≃+* Rᵒᵖ} {G : sesq_form R M K} {x y : M} {a : R} (ha : a 0) :
G.is_ortho x y G.is_ortho (a x) y

theorem sesq_form.ortho_smul_right {R : Type u_1} [domain R] {M : Type v} [add_comm_group M] [module R M] {K : R ≃+* Rᵒᵖ} {G : sesq_form R M K} {x y : M} {a : R} (ha : a 0) :
G.is_ortho x y G.is_ortho x (a y)

def refl_sesq_form.is_refl {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} (S : sesq_form R M I) :
Prop

The proposition that a sesquilinear form is reflexive

Equations
theorem refl_sesq_form.eq_zero {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : refl_sesq_form.is_refl S) {x y : M} (a : S x y = 0) :
S y x = 0

theorem refl_sesq_form.ortho_sym {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : refl_sesq_form.is_refl S) {x y : M} :
S.is_ortho x y S.is_ortho y x

def sym_sesq_form.is_sym {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} (S : sesq_form R M I) :
Prop

The proposition that a sesquilinear form is symmetric

Equations
theorem sym_sesq_form.sym {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : sym_sesq_form.is_sym S) (x y : M) :
opposite.unop (I (S x y)) = S y x

theorem sym_sesq_form.is_refl {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : sym_sesq_form.is_sym S) :

theorem sym_sesq_form.ortho_sym {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : sym_sesq_form.is_sym S) {x y : M} :
S.is_ortho x y S.is_ortho y x

def alt_sesq_form.is_alt {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} (S : sesq_form R M I) :
Prop

The proposition that a sesquilinear form is alternating

Equations
theorem alt_sesq_form.self_eq_zero {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : alt_sesq_form.is_alt S) (x : M) :
S x x = 0

theorem alt_sesq_form.neg {R : Type u_1} {M : Type u_2} [ring R] [add_comm_group M] [module R M] {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I} (H : alt_sesq_form.is_alt S) (x y : M) :
-S x y = S y x