Skip to content

Conversation

@vihdzp
Copy link
Collaborator

@vihdzp vihdzp commented Sep 15, 2025

@github-actions
Copy link

github-actions bot commented Sep 15, 2025

PR summary 89423f926a

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.Algebra.Order.Ring.StandardPart (new file) 1349

Declarations diff

+ FiniteElement
+ FiniteResidueField
+ ext
+ ind
+ instLinearOrder
+ instance : Archimedean (FiniteResidueField K)
+ instance : CommRing (FiniteElement K) := by
+ instance : Field (FiniteResidueField K)
+ instance : IsDomain (FiniteElement K) := by
+ instance : IsOrderedRing (FiniteResidueField K)
+ instance : IsStrictOrderedRing (FiniteElement K) := by
+ instance : LinearOrder (FiniteElement K) := by
+ instance : LinearOrder (FiniteResidueField K)
+ instance : ValuationRing (FiniteElement K) := by
+ isUnit_iff_mk_eq_zero
+ lt_of_mk_lt_mk
+ mk_eq_mk
+ mk_eq_zero
+ mk_intCast
+ mk_le_add_mk_of_archimedean
+ mk_le_mk
+ mk_le_mk_add_of_archimedean
+ mk_lt_mk
+ mk_map_nonneg_of_archimedean
+ mk_natCast
+ mk_ne_zero
+ mk_neg
+ mk_one
+ mk_sub_pos_iff
+ mk_sub_stdPart_pos
+ mk_zero
+ not_isUnit_iff_mk_pos
+ ofArchimedean
+ ofArchimedean_apply
+ ofArchimedean_inj
+ ofArchimedean_injective
+ ofArchimedean_stdPart
+ ordConnected_preimage_mk
+ stdPart
+ stdPart_add
+ stdPart_div
+ stdPart_intCast
+ stdPart_inv
+ stdPart_mul
+ stdPart_natCast
+ stdPart_neg
+ stdPart_ofNat
+ stdPart_of_mk_ne_zero
+ stdPart_of_mk_nonneg
+ stdPart_one
+ stdPart_ratCast
+ stdPart_real
+ stdPart_sub
+ stdPart_zero
+ val_add
+ val_mul
+ val_one
+ val_sub
+ val_zero
++ mk
- instance [DecidableRel (· ≈ · : α → α → Prop)] : LinearOrder (Quotient s)

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

@vihdzp vihdzp marked this pull request as draft September 16, 2025 00:28
@mathlib4-merge-conflict-bot mathlib4-merge-conflict-bot added the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Sep 24, 2025
@mathlib4-merge-conflict-bot
Copy link
Collaborator

This pull request has conflicts, please merge master and resolve them.

@vihdzp vihdzp removed the awaiting-author A reviewer has asked the author a question or requested changes. label Dec 15, 2025
@YaelDillies YaelDillies added the awaiting-author A reviewer has asked the author a question or requested changes. label Dec 15, 2025
@vihdzp vihdzp removed the awaiting-author A reviewer has asked the author a question or requested changes. label Dec 15, 2025
Copy link
Collaborator

@YaelDillies YaelDillies left a comment

Choose a reason for hiding this comment

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

Thanks! 🚀

maintainer merge

@github-actions
Copy link

🚀 Pull request has been placed on the maintainer queue by YaelDillies.

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. label Dec 15, 2025
Comment on lines +222 to +223
/-- The standard part of a `FiniteElement` is the unique real number with an infinitesimal
difference.
Copy link
Member

Choose a reason for hiding this comment

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

Can you add that as a lemma characterizing this def?

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 had that on a follow-up PR, but I can move it here.

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

Just added this theorem, along with some prerequisite lemmas.

@jcommelin jcommelin added awaiting-author A reviewer has asked the author a question or requested changes. and removed maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. labels Dec 16, 2025
@vihdzp vihdzp removed the awaiting-author A reviewer has asked the author a question or requested changes. label Dec 16, 2025
Copy link
Member

@jcommelin jcommelin 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 Dec 17, 2025
mathlib-bors bot pushed a commit that referenced this pull request Dec 17, 2025
We define `ArchimedeanClass.stdPart x` as the unique real number with an infinitesimal difference from `x`. This generalizes `Hyperreal.st` for a general (non-)archimedean field.

Co-authored-by: pre-commit-ci-lite[bot] <117423508+pre-commit-ci-lite[bot]@users.noreply.github.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Dec 17, 2025

Build failed (retrying...):

mathlib-bors bot pushed a commit that referenced this pull request Dec 17, 2025
We define `ArchimedeanClass.stdPart x` as the unique real number with an infinitesimal difference from `x`. This generalizes `Hyperreal.st` for a general (non-)archimedean field.

Co-authored-by: pre-commit-ci-lite[bot] <117423508+pre-commit-ci-lite[bot]@users.noreply.github.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Dec 17, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feat: standard part in non-Archimedean field [Merged by Bors] - feat: standard part in non-Archimedean field Dec 17, 2025
@mathlib-bors mathlib-bors bot closed this Dec 17, 2025
YuvalFilmus pushed a commit to YuvalFilmus/mathlib4 that referenced this pull request Dec 19, 2025
)

We define `ArchimedeanClass.stdPart x` as the unique real number with an infinitesimal difference from `x`. This generalizes `Hyperreal.st` for a general (non-)archimedean field.

Co-authored-by: pre-commit-ci-lite[bot] <117423508+pre-commit-ci-lite[bot]@users.noreply.github.com>
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-algebra Algebra (groups, rings, fields, etc)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

9 participants