Skip to content

Conversation

themathqueen
Copy link
Collaborator

@themathqueen themathqueen commented Jul 15, 2025

For symmetric projections p and q, p ≤ q iff range p ≤ range q, so then: U.starProjection ≤ V.starProjection iff U ≤ V, which implies that Submodule.starProjection is an injective function.


Open in Gitpod

@j-loreaux j-loreaux added the awaiting-author A reviewer has asked the author a question or requested changes. label Sep 23, 2025
@themathqueen themathqueen removed the awaiting-author A reviewer has asked the author a question or requested changes. label Sep 23, 2025
Comment on lines 323 to 334
theorem IsSymmetricProjection.sub_of_comp_eq_right {p q : E →ₗ[𝕜] E}
(hp : p.IsSymmetricProjection) (hq : q.IsSymmetricProjection) (hqp : q ∘ₗ p = p) :
(q - p).IsSymmetricProjection := by
refine ⟨hp.isIdempotentElem.sub hq.isIdempotentElem (LinearMap.ext fun x => ext_inner_left 𝕜
fun y => ?_) hqp, hq.isSymmetric.sub hp.isSymmetric⟩
simp_rw [Module.End.mul_apply, ← hp.isSymmetric _, ← hq.isSymmetric _, ← comp_apply, hqp]

theorem IsSymmetricProjection.sub_of_comp_eq_left {p q : E →ₗ[𝕜] E}
(hp : p.IsSymmetricProjection) (hq : q.IsSymmetricProjection) (hpq : p ∘ₗ q = p) :
(q - p).IsSymmetricProjection := by
refine hp.sub_of_comp_eq_right hq <| LinearMap.ext fun x => ext_inner_left 𝕜 fun y => ?_
simp_rw [comp_apply, ← hq.isSymmetric _, ← hp.isSymmetric _, ← comp_apply, hpq]
Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

@j-loreaux, should we just have one version of this instead as well?
IsSymmetricProjection.sub_of_range_le_range: range p ≤ range q implies q - p is a symmetric projection?

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I changed it, let me know if I should change it back

@j-loreaux j-loreaux added the awaiting-author A reviewer has asked the author a question or requested changes. label Sep 23, 2025
@themathqueen themathqueen removed the awaiting-author A reviewer has asked the author a question or requested changes. label Oct 17, 2025
Copy link
Collaborator

@j-loreaux j-loreaux left a comment

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Thanks

bors merge

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the ready-to-merge This PR has been sent to bors. label Oct 18, 2025
mathlib-bors bot pushed a commit that referenced this pull request Oct 18, 2025
…Projection` iff `U ≤ V` (#27162)

For symmetric projections `p` and `q`, `p ≤ q` iff `range p ≤ range q`, so then: `U.starProjection ≤ V.starProjection` iff `U ≤ V`, which implies that `Submodule.starProjection` is an injective function.
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Oct 18, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feat(Analysis/InnerProductSpace/Positive): U.starProjection ≤ V.starProjection iff U ≤ V [Merged by Bors] - feat(Analysis/InnerProductSpace/Positive): U.starProjection ≤ V.starProjection iff U ≤ V Oct 18, 2025
@mathlib-bors mathlib-bors bot closed this Oct 18, 2025
@themathqueen themathqueen deleted the starProjection_le branch October 18, 2025 20:49
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

ready-to-merge This PR has been sent to bors. t-analysis Analysis (normed *, calculus)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

7 participants