Positive operators #
In this file we define when an operator in a Hilbert space is positive. We follow Bourbaki's choice of requiring self adjointness in the definition.
Main definitions #
LinearMap.IsPositive
: a linear map is positive if it is self adjoint and∀ x, 0 ≤ re ⟪T x, x⟫
.ContinuousLinearMap.IsPositive
: a continuous linear map is positive if it is self adjoint and∀ x, 0 ≤ re ⟪T x, x⟫
.
Main statements #
ContinuousLinearMap.IsPositive.conj_adjoint
: ifT : E →L[𝕜] E
is positive, then for anyS : E →L[𝕜] F
,S ∘L T ∘L S†
is also positive.ContinuousLinearMap.isPositive_iff_complex
: in a complex Hilbert space, checking that⟪T x, x⟫
is a nonnegative real number for allx
suffices to prove thatT
is positive.
References #
Tags #
Positive operator
A continuous linear endomorphism T
of a Hilbert space is positive if it is self adjoint
and ∀ x, 0 ≤ re ⟪T x, x⟫
.
Equations
- T.IsPositive = (IsSelfAdjoint T ∧ ∀ (x : E), 0 ≤ T.reApplyInnerSelf x)
Instances For
The (Loewner) partial order on continuous linear maps on a Hilbert space determined by
f ≤ g
if and only if g - f
is a positive linear map (in the sense of
ContinuousLinearMap.IsPositive
). With this partial order, the continuous linear maps form a
StarOrderedRing
.
Equations
- ContinuousLinearMap.instLoewnerPartialOrder = { le := fun (f g : E →L[𝕜] E) => (g - f).IsPositive, le_refl := ⋯, le_trans := ⋯, lt_iff_le_not_ge := ⋯, le_antisymm := ⋯ }
A linear map T
of a Hilbert space is positive if it is self adjoint and
∀ x, 0 ≤ re ⟪T x, x⟫
.
Equations
- T.IsPositive = (IsSelfAdjoint T ∧ ∀ (x : E), 0 ≤ RCLike.re (inner 𝕜 (T x) x))
Instances For
The (Loewner) partial order on linear maps on a Hilbert space determined by f ≤ g
if and only if g - f
is a positive linear map (in the sense of LinearMap.IsPositive
).
Equations
- LinearMap.instLoewnerPartialOrder = { le := fun (f g : E →ₗ[𝕜] E) => (g - f).IsPositive, le_refl := ⋯, le_trans := ⋯, lt_iff_le_not_ge := ⋯, le_antisymm := ⋯ }