Skip to content

Conversation

@tdwag123
Copy link

@tdwag123 tdwag123 commented Dec 13, 2025

feat(MeasureTheory/Measure/TypeClass/NoAtoms): Added a theorem that states If a set has positive measure under an atomless measure, then it has an accumulation point.

Added a lemma in (Topology/DiscreteSubset): If a subset of a topological space has no accumulation points,
then it carries the discrete topology.

Theorem added: exists_accPt_of_pos_hausdorffMeasure
Lemma added: discreteTopology_of_noAccPts

Harmonic's Aristotle gave the initial version of the proofs. I did substantial work shortening the proof from 40 lines and refactoring it into another Lemma.

Special thanks to @plp127 and @CoolRmal for the useful feedback in the PR process.

**Co-authored-by: @Aristotle-Harmonic **

---

Open in Gitpod

Added a theorem that states if a set has positive s-dimensional Hausdorff measure, then it has an accumulation point, along with necessary proofs.
feat(MeasureTheory/Measure/Hausdorff)  ∀ 𝑠 > 0, ∀ 𝐸 ⊂ 𝑅^𝑛, 𝐻^𝑠 (𝐸)>0 ⇒ ∃ 𝑥 ∈ 𝑅^𝑛 , 𝑥 is an accumulation point of 𝑃(𝐸).
@github-actions github-actions bot added the new-contributor This PR was made by a contributor with at most 5 merged PRs. Welcome to the community! label Dec 13, 2025
@github-actions github-actions bot added the t-measure-probability Measure theory / Probability theory label Dec 13, 2025
@github-actions
Copy link

github-actions bot commented Dec 13, 2025

PR summary 98379c78c5

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ discreteTopology_of_noAccPts
+ exists_accPt_of_noAtoms

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
Copy link

github-actions bot commented Dec 13, 2025

🚨 PR Title Needs Formatting

Please update the title to match our commit style conventions.

Errors from script:

error: the PR title does not contain a colon
Details on the required title format

The title should fit the following format:

<kind>(<optional-scope>): <subject>

<kind> is:

  • feat (feature)
  • fix (bug fix)
  • doc (documentation)
  • style (formatting, missing semicolons, ...)
  • refactor
  • test (when adding missing tests)
  • chore (maintain)
  • perf (performance improvement, optimization, ...)
  • ci (changes to continuous integration, repo automation, ...)

<optional-scope> is a name of module or a directory which contains changed modules.
This is not necessary to include, but may be useful if the <subject> is insufficient.
The Mathlib directory prefix is always omitted.
For instance, it could be

  • Data/Nat/Basic
  • Algebra/Group/Defs
  • Topology/Constructions

<subject> has the following constraints:

  • do not capitalize the first letter
  • no dot(.) at the end
  • use imperative, present tense: "change" not "changed" nor "changes"

@tdwag123 tdwag123 marked this pull request as draft December 13, 2025 20:13
tdwag123 and others added 2 commits December 13, 2025 12:17
I removed the simp using simp? to find the appropriate simp only statement
@tdwag123 tdwag123 marked this pull request as ready for review December 13, 2025 20:36
Refactor the theorem to use a more general type for the set and include separability condition. I tried to take into account the suggestions, but I may have missed some. The theorem needed some bigger reworking after the generalization
generalization and change of location

Added a theorem to show that if a set has positive measure under an atomless measure, then it has an accumulation point.
Added lemma for discrete topology based on no accumulation points.
Introduce lemma for discrete topology with no AccPts
@tdwag123 tdwag123 requested a review from plp127 December 21, 2025 05:12
@plp127
Copy link
Collaborator

plp127 commented Dec 21, 2025

Can you update the PR title and description?

@tdwag123 tdwag123 changed the title feat(MeasureTheory/Measure/Hausdorff) add exists_accPt_of_pos_hausdorffMeasure feat(MeasureTheory/Measure/TypeClass/NoAtoms) add exists_accPt_of_noAtoms Dec 21, 2025
Removed lemma about discrete topology for sets with no accumulation points.
@tdwag123 tdwag123 requested a review from CoolRmal December 27, 2025 02:13
Copy link
Contributor

@CoolRmal CoolRmal left a comment

Choose a reason for hiding this comment

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

I think this is ready to be merged after some minor changes.

@sgouezel
Copy link
Contributor

Could you close the discussions for which you think they have been dealt with? It helps the reviewers to see what remains to be done.

tdwag123 and others added 4 commits December 27, 2025 17:20
Co-authored-by: Yongxi (Aaron) Lin <97214596+CoolRmal@users.noreply.github.com>
Co-authored-by: Yongxi (Aaron) Lin <97214596+CoolRmal@users.noreply.github.com>
Moved out of the partial ordering section, factored some variables out the `exists_accPt_of_noAtoms ` theorem
added section wrappers around the theorem to prevent issues with `μ : Measure α` versus the partial measure `α`
@sgouezel sgouezel added the awaiting-author A reviewer has asked the author a question or requested changes. label Jan 2, 2026
tdwag123 and others added 4 commits January 7, 2026 23:54
Refactor the `exists_accPt_of_noAtoms` theorem for clarity and structure.

-Removed the section for the theorem
-Changed the assumptions to make them weaker
-Changed where the open statements are

Still to be done:
See if I can refactor and make the assumptions even weaker.
Changed the assumptions for `exists_accPt_of_noAtoms` from [EPseudometricSpace] to [TopologicalSpace X]
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

awaiting-author A reviewer has asked the author a question or requested changes. new-contributor This PR was made by a contributor with at most 5 merged PRs. Welcome to the community! t-measure-probability Measure theory / Probability theory

Projects

None yet

Development

Successfully merging this pull request may close these issues.

6 participants