Documentation

Mathlib.Analysis.InnerProductSpace.JointEigenspace

Joint eigenspaces of a commuting pair of symmetric operators #

This file collects various decomposition results for joint eigenspaces of a commuting pair of symmetric operators on a finite-dimensional inner product space.

Main Result #

TODO #

Develop a Diagonalization structure for linear maps and / or matrices which consists of a basis, and a proof obligation that the basis vectors are eigenvectors.

Tags #

self-adjoint operator, simultaneous eigenspaces, joint eigenspaces

theorem LinearMap.IsSymmetric.eigenspace_invariant_of_commute {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} (hAB : A โˆ˜โ‚— B = B โˆ˜โ‚— A) (ฮฑ : ๐•œ) (v : E) :

If a pair of operators commute, then the eigenspaces of one are invariant under the other.

theorem LinearMap.IsSymmetric.orthogonalFamily_eigenspace_inf_eigenspace {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} (hA : A.IsSymmetric) (hB : B.IsSymmetric) :
OrthogonalFamily ๐•œ (fun (i : ๐•œ ร— ๐•œ) => { x : E // x โˆˆ Module.End.eigenspace A i.2 โŠ“ Module.End.eigenspace B i.1 }) fun (i : ๐•œ ร— ๐•œ) => (Module.End.eigenspace A i.2 โŠ“ Module.End.eigenspace B i.1).subtypeโ‚—แตข

The simultaneous eigenspaces of a pair of commuting symmetric operators form an OrthogonalFamily.

theorem LinearMap.IsSymmetric.eigenspace_inf_eigenspace {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {ฮฑ : ๐•œ} {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} (hAB : A โˆ˜โ‚— B = B โˆ˜โ‚— A) (ฮณ : ๐•œ) :
Module.End.eigenspace A ฮฑ โŠ“ Module.End.eigenspace B ฮณ = Submodule.map (Module.End.eigenspace A ฮฑ).subtype (Module.End.eigenspace (B.restrict โ‹ฏ) ฮณ)

The intersection of eigenspaces of commuting selfadjoint operators is equal to the eigenspace of one operator restricted to the eigenspace of the other, which is an invariant subspace because the operators commute.

theorem LinearMap.IsSymmetric.iSup_eigenspace_inf_eigenspace {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {ฮฑ : ๐•œ} {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} [FiniteDimensional ๐•œ E] (hB : B.IsSymmetric) (hAB : A โˆ˜โ‚— B = B โˆ˜โ‚— A) :
โจ† (ฮณ : ๐•œ), Module.End.eigenspace A ฮฑ โŠ“ Module.End.eigenspace B ฮณ = Module.End.eigenspace A ฮฑ

If A and B are commuting symmetric operators on a finite dimensional inner product space then the eigenspaces of the restriction of B to any eigenspace of A exhaust that eigenspace.

theorem LinearMap.IsSymmetric.iSup_iSup_eigenspace_inf_eigenspace_eq_top {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} [FiniteDimensional ๐•œ E] (hA : A.IsSymmetric) (hB : B.IsSymmetric) (hAB : A โˆ˜โ‚— B = B โˆ˜โ‚— A) :
โจ† (ฮฑ : ๐•œ), โจ† (ฮณ : ๐•œ), Module.End.eigenspace A ฮฑ โŠ“ Module.End.eigenspace B ฮณ = โŠค

If A and B are commuting symmetric operators acting on a finite dimensional inner product space, then the simultaneous eigenspaces of A and B exhaust the space.

theorem LinearMap.IsSymmetric.directSum_isInteral_of_commute {๐•œ : Type u_1} {E : Type u_2} [RCLike ๐•œ] [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] {A : E โ†’โ‚—[๐•œ] E} {B : E โ†’โ‚—[๐•œ] E} [FiniteDimensional ๐•œ E] (hA : A.IsSymmetric) (hB : B.IsSymmetric) (hAB : A โˆ˜โ‚— B = B โˆ˜โ‚— A) :

Given a commuting pair of symmetric linear operators on a finite dimensional inner product space, the space decomposes as an internal direct sum of simultaneous eigenspaces of these operators.