Skip to content

Commit

Permalink
feat: add the Loewner partial order on continuous linear maps on a Hi…
Browse files Browse the repository at this point in the history
…lbert space (#12026)

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`.
  • Loading branch information
j-loreaux committed Apr 9, 2024
1 parent e8433a6 commit b5b45d3
Showing 1 changed file with 30 additions and 0 deletions.
30 changes: 30 additions & 0 deletions Mathlib/Analysis/InnerProductSpace/Positive.lean
Expand Up @@ -125,4 +125,34 @@ theorem isPositive_iff_complex (T : E' →L[ℂ] E') :

end Complex

section PartialOrder

/-- 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`. -/
instance instLoewnerPartialOrder : PartialOrder (E →L[𝕜] E) where
le f g := (g - f).IsPositive
le_refl _ := by simpa using isPositive_zero
le_trans _ _ _ h₁ h₂ := by simpa using h₁.add h₂
le_antisymm f₁ f₂ h₁ h₂ := by
rw [← sub_eq_zero]
have h_isSymm := isSelfAdjoint_iff_isSymmetric.mp h₂.isSelfAdjoint
exact_mod_cast h_isSymm.inner_map_self_eq_zero.mp fun x ↦ by
apply RCLike.ext
· rw [map_zero]
apply le_antisymm
· rw [← neg_nonneg, ← map_neg, ← inner_neg_left]
simpa using h₁.inner_nonneg_left _
· exact h₂.inner_nonneg_left _
· rw [coe_sub, LinearMap.sub_apply, coe_coe, coe_coe, map_zero, ← sub_apply,
← h_isSymm.coe_reApplyInnerSelf_apply (T := f₁ - f₂) x, RCLike.ofReal_im]

lemma le_def (f g : E →L[𝕜] E) : f ≤ g ↔ (g - f).IsPositive := Iff.rfl

lemma nonneg_iff_isPositive (f : E →L[𝕜] E) : 0 ≤ f ↔ f.IsPositive := by
simpa using le_def 0 f

end PartialOrder

end ContinuousLinearMap

0 comments on commit b5b45d3

Please sign in to comment.