Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

[Merged by Bors] - split(topology/algebra/infinite_sum): Split into four files #18414

Closed
wants to merge 7 commits into from

Conversation

YaelDillies
Copy link
Collaborator

@YaelDillies YaelDillies commented Feb 9, 2023

Over the past five years, topology.algebra.infinite_sum has grown pretty big. This PR splits off a third of it to three new files. Precisely, split topology.algebra.infinite_sum into:

Incidentally, this brings down some files' imports by quite a lot.

Also move the star and mul_opposite material to the end of the file to facilitate multiplicativisation in #18405.

Johannes wrote some of all these files, except topology.algebra.infinite_sum.real whose first lemma I could trace back as coming from #753, with the others coming from #1739.


Partially requested by @eric-wieser

Open in Gitpod

@YaelDillies YaelDillies requested a review from a team as a code owner February 9, 2023 21:17
@YaelDillies YaelDillies added awaiting-CI The author would like to see what CI has to say before doing more work. awaiting-review The author would like community review of the PR t-algebra Algebra (groups, rings, fields etc) t-order Order hierarchy t-topology Topological spaces, uniform spaces, metric spaces, filters labels Feb 9, 2023
@eric-wieser
Copy link
Member

  • topology.algebra.big_operators.ring: Interaction of infinite sums and (scalar) multiplication. This cannot be multiplicativised.

mul_distrib_mul_action and mul_semiring_action are arguably counterexamples to this claim

@eric-wieser
Copy link
Member

(I didn't request a split, only a reorder; but I'm not opposed either)

@YaelDillies
Copy link
Collaborator Author

YaelDillies commented Feb 9, 2023

  • topology.algebra.big_operators.ring: Interaction of infinite sums and (scalar) multiplication. This cannot be multiplicativised.

mul_distrib_mul_action and mul_semiring_action are arguably counterexamples to this claim

Do you think this changes the way these files should be split? Note that it's not enough to have mul_distrib_mul_action and mul_semiring_action. We need ways to state they act continuously. I think has_continuous_const_smul provides this assumption for a few lemmas, but I doubt the other required one exists.

Copy link
Member

@eric-wieser eric-wieser left a comment

Choose a reason for hiding this comment

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

This split generally looks reasonable to me. My main comments would be:

  • infinite_sum might be preferable to big_operators as a name; it doesn't matter to me, but might to other reviewers
  • topology.algebra.module.infinite_sum feels out of place now that the other file is not called infinite_sum.
  • I'm not convinced about the placement of the smul lemmas, but that's minor.
  • The docstrings of (some) of the new files could maybe do with a "main results" section.

@github-actions github-actions bot removed the awaiting-CI The author would like to see what CI has to say before doing more work. label Feb 9, 2023
@YaelDillies
Copy link
Collaborator Author

  • I am reluctant to keeping infinite_sum as a name given that we're about to acquire infinite products in the same files. But I'd gladly take opinions
  • Moved
  • Moved
  • I've expanded a bit for topology.algebra.big_operators.ring, but I have no idea about the other ones.

@eric-wieser eric-wieser changed the title split(topology/algebra/big_operators/*): Split into four files split(topology/algebra/infinite_sum): Split into four files and rename to big_operators Feb 11, 2023
@eric-wieser eric-wieser changed the title split(topology/algebra/infinite_sum): Split into four files and rename to big_operators refactor(topology/algebra/infinite_sum): Split into four files and rename to big_operators Feb 11, 2023
@YaelDillies YaelDillies changed the title refactor(topology/algebra/infinite_sum): Split into four files and rename to big_operators split(topology/algebra/infinite_sum): Split into four files Feb 15, 2023
Copy link
Member

@eric-wieser eric-wieser 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+

Thanks!

@bors
Copy link

bors bot commented Feb 15, 2023

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

@leanprover-community-bot-assistant leanprover-community-bot-assistant added delegated The PR author may merge after reviewing final suggestions. and removed awaiting-review The author would like community review of the PR labels Feb 15, 2023
@YaelDillies
Copy link
Collaborator Author

bors merge

bors bot pushed a commit that referenced this pull request Feb 15, 2023
Over the past five years, `topology.algebra.infinite_sum` has grown pretty big. This PR splits off a third of it to three new files. Precisely, split `topology.algebra.infinite_sum` into:
* `topology.algebra.infinite_sum.basic`: Definitions and theory in monoids. All this will be multiplicativised in #18405.
* `topology.algebra.infinite_sum.ring`: Interaction of infinite sums and (scalar) multiplication. This mostly cannot be multiplicativised.
* `topology.algebra.infinite_sum.order`: Interaction of infinite sums and order. Most of this will be multiplicativised in #18405.

Incidentally, this brings down some files' imports by quite a lot.

Also move the `star` and `mul_opposite` material to the end of the file to facilitate multiplicativisation in #18405.

Johannes wrote some of all these files, except `topology.algebra.infinite_sum.real` whose first lemma I could trace back as coming from #753, with the others coming from #1739.
@bors
Copy link

bors bot commented Feb 15, 2023

Build failed:

@YaelDillies
Copy link
Collaborator Author

bors merge

bors bot pushed a commit that referenced this pull request Feb 15, 2023
Over the past five years, `topology.algebra.infinite_sum` has grown pretty big. This PR splits off a third of it to three new files. Precisely, split `topology.algebra.infinite_sum` into:
* `topology.algebra.infinite_sum.basic`: Definitions and theory in monoids. All this will be multiplicativised in #18405.
* `topology.algebra.infinite_sum.ring`: Interaction of infinite sums and (scalar) multiplication. This mostly cannot be multiplicativised.
* `topology.algebra.infinite_sum.order`: Interaction of infinite sums and order. Most of this will be multiplicativised in #18405.

Incidentally, this brings down some files' imports by quite a lot.

Also move the `star` and `mul_opposite` material to the end of the file to facilitate multiplicativisation in #18405.

Johannes wrote some of all these files, except `topology.algebra.infinite_sum.real` whose first lemma I could trace back as coming from #753, with the others coming from #1739.
@bors
Copy link

bors bot commented Feb 15, 2023

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title split(topology/algebra/infinite_sum): Split into four files [Merged by Bors] - split(topology/algebra/infinite_sum): Split into four files Feb 15, 2023
@bors bors bot closed this Feb 15, 2023
@bors bors bot deleted the split_tsum branch February 15, 2023 19:45
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
delegated The PR author may merge after reviewing final suggestions. t-algebra Algebra (groups, rings, fields etc) t-order Order hierarchy t-topology Topological spaces, uniform spaces, metric spaces, filters
Projects
None yet
Development

Successfully merging this pull request may close these issues.

3 participants