Skip to content

Conversation

mans0954
Copy link
Collaborator

@mans0954 mans0954 commented Sep 2, 2025

Let R and A be ordered rings, A an R-algebra and R, A, M a scalar tower. We provide sufficient conditions for an R-convex subset of M to be A-convex and for an A-convex subset of M to be R-convex.

These are used to show that, when K is RCLike and K E is a scalar tower, a set is K-convex if and only if it is -convex.

Used in #29258


Open in Gitpod

@mans0954 mans0954 added the WIP Work in progress label Sep 2, 2025
@github-actions github-actions bot added the t-analysis Analysis (normed *, calculus) label Sep 2, 2025
Copy link

github-actions bot commented Sep 2, 2025

PR summary 6549fa3760

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ convex_RCLike_iff_convex_real
+ convex_of_nonneg_surjective_algebraMap

You can run this locally as follows
## summary with just the declaration names:
./scripts/declarations_diff.sh <optional_commit>

## more verbose report:
./scripts/declarations_diff.sh long <optional_commit>

The doc-module for script/declarations_diff.sh contains some details about this script.


No changes to technical debt.

You can run this locally as

./scripts/technical-debt-metrics.sh pr_summary
  • The relative value is the weighted sum of the differences with weight given by the inverse of the current value of the statistic.
  • The absolute value is the relative value divided by the total sum of the inverses of the current values (i.e. the weighted average of the differences).

@mans0954 mans0954 marked this pull request as ready for review September 2, 2025 17:07
@mans0954
Copy link
Collaborator Author

mans0954 commented Sep 2, 2025

The proof is inspired by Convex.convex_isRCLikeNormedField - but I couldn't find a way to deduce Convex.convex_isRCLikeNormedField from convex_of_nonneg_algebraMap.

@mans0954 mans0954 removed the WIP Work in progress label Sep 2, 2025
@mans0954
Copy link
Collaborator Author

mans0954 commented Sep 4, 2025

c.f. #29075

@mans0954
Copy link
Collaborator Author

mans0954 commented Sep 4, 2025

CC: @Timeroot - any thoughts on this PR please?

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.

Certainly this seems useful, but I'm a bit unclear about the supposed extra generality.

I would like to switch some statements about Hahn-Banach to use LocallyConvexSpace 𝕜 E instead of LocallyConvexSpace ℝ E with this.

@j-loreaux j-loreaux added the awaiting-author A reviewer has asked the author a question or requested changes. label Sep 30, 2025
@mans0954
Copy link
Collaborator Author

mans0954 commented Oct 1, 2025

Certainly this seems useful, but I'm a bit unclear about the supposed extra generality.

@j-loreaux it's an artifact of me starting this PR before I was aware of #29075 - I've removed the unnecessary extra generality now.

I would like to switch some statements about Hahn-Banach to use LocallyConvexSpace 𝕜 E instead of LocallyConvexSpace ℝ E with this.

You might also be interested in #29342 which sorts out an awkward work-around in the definition of AbsConvex.

@mans0954 mans0954 removed the awaiting-author A reviewer has asked the author a question or requested changes. label Oct 1, 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.

bors merge

variable {M : Type*} [AddCommMonoid M] [Module A M] [Module R M] [IsScalarTower R A M]
variable [PartialOrder R] [PartialOrder A]

lemma convex_of_nonneg_surjective_algebraMap [FaithfulSMul R A] {s : Set M}
Copy link
Collaborator

Choose a reason for hiding this comment

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

The name of this declaration is a little misleading as Function.Surjective does not appear, but I think it's a niche enough result that I'm not going to quibble further.

mathlib-bors bot pushed a commit that referenced this pull request Oct 2, 2025
Let `R` and `A` be ordered rings, `A` an `R`-algebra and `R`, `A`, `M` a scalar tower. We provide sufficient conditions for an `R`-convex subset of `M` to be `A`-convex and for an `A`-convex subset of `M` to be `R`-convex.

These are used to show that, when `K` is `RCLike` and `ℝ` `K` `E` is a scalar tower, a set is `K`-convex if and only if it is `ℝ`-convex.

Used in #29258
@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the ready-to-merge This PR has been sent to bors. label Oct 2, 2025
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Oct 2, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feature(Analysis/Convex/Basic): Convexity and the algebra map [Merged by Bors] - feature(Analysis/Convex/Basic): Convexity and the algebra map Oct 2, 2025
@mathlib-bors mathlib-bors bot closed this Oct 2, 2025
mitchell-horner pushed a commit to mitchell-horner/mathlib4 that referenced this pull request Oct 6, 2025
…over-community#29248)

Let `R` and `A` be ordered rings, `A` an `R`-algebra and `R`, `A`, `M` a scalar tower. We provide sufficient conditions for an `R`-convex subset of `M` to be `A`-convex and for an `A`-convex subset of `M` to be `R`-convex.

These are used to show that, when `K` is `RCLike` and `ℝ` `K` `E` is a scalar tower, a set is `K`-convex if and only if it is `ℝ`-convex.

Used in leanprover-community#29258
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.

3 participants