Skip to content

Conversation

erdOne
Copy link
Member

@erdOne erdOne commented Oct 10, 2025


Open in Gitpod

@github-actions github-actions bot added the large-import Automatically added label for PRs with a significant increase in transitive imports label Oct 10, 2025
Copy link

github-actions bot commented Oct 10, 2025

PR summary 1f85fdff73

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ instance : PathConnectedSpace ℂˣ

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).

@github-actions github-actions bot added the t-analysis Analysis (normed *, calculus) label Oct 10, 2025
@erdOne erdOne force-pushed the erd1/pathconnectedC branch from f13caa4 to 18823bb Compare October 10, 2025 20:37
@github-actions github-actions bot removed the large-import Automatically added label for PRs with a significant increase in transitive imports label Oct 10, 2025
Co-authored-by: Aaron Liu <aaronliu2008@outlook.com>
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 d+

Rectangle z w ⊆ U := by
simpa only [rectangle_eq_convexHull] using convexHull_min (by grind) U_convex

instance : PathConnectedSpace ℂˣ :=
Copy link
Collaborator

Choose a reason for hiding this comment

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

Please add a comment explaining that this could be proved faster using other means (e.g., via the exponential map, or via facts about real vector spaces of dimension exceeding one), but that this approach was adopted to minimize imports.

@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Oct 18, 2025

✌️ erdOne can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

@Komyyy
Copy link
Collaborator

Komyyy commented Oct 18, 2025

I think this proof can be golfed using isPathConnected_compl_singleton_of_one_lt_rank.

@erdOne
Copy link
Member Author

erdOne commented Oct 18, 2025

Yes but it requires a lot more import. But this is a valid point and is also what Jireh has suggested.

@Komyyy
Copy link
Collaborator

Komyyy commented Oct 18, 2025

Sorry, I didn't read @j-loreaux 's comments, please forget.

@erdOne
Copy link
Member Author

erdOne commented Oct 18, 2025

bors merge

mathlib-bors bot pushed a commit that referenced this pull request Oct 18, 2025
@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): PathConnectedSpace ℂˣ [Merged by Bors] - feat(Analysis): PathConnectedSpace ℂˣ Oct 18, 2025
@mathlib-bors mathlib-bors bot closed this Oct 18, 2025
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

delegated t-analysis Analysis (normed *, calculus)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

5 participants