Skip to content

Conversation

@vihdzp
Copy link
Collaborator

@vihdzp vihdzp commented Dec 30, 2025

Used in the CGT repo.


I don't know if it's possible to relax Ring to Semiring.

Open in Gitpod

@vihdzp vihdzp requested a review from wwylele December 30, 2025 08:48
@github-actions github-actions bot added the large-import Automatically added label for PRs with a significant increase in transitive imports label Dec 30, 2025
@github-actions
Copy link

github-actions bot commented Dec 30, 2025

PR summary ce5b0921e0

Import changes exceeding 2%

% File
+32.41% Mathlib.RingTheory.HahnSeries.Lex

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.RingTheory.HahnSeries.Lex 651 862 +211 (+32.41%)
Import changes for all files
Files Import difference
Mathlib.RingTheory.HahnSeries.HahnEmbedding 6
Mathlib.Algebra.Order.Module.HahnEmbedding 57
Mathlib.RingTheory.HahnSeries.Lex 211

Declarations diff

+ instance [IsOrderedRing R] [NoZeroDivisors R] : IsOrderedRing (Lex R⟦Γ⟧)
+ instance [IsStrictOrderedRing R] : IsStrictOrderedRing (Lex R⟦Γ⟧)
+ leadingCoeff_mul
+ leadingCoeff_mul_of_ne_zero
+ orderTop_mul
+ orderTop_mul_of_ne_zero
+ order_mul_of_ne_zero

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.


Decrease in tech debt: (relative, absolute) = (1.00, 0.01)
Current number Change Type
143 -1 flexible linter exceptions

Current commit b2622002b7
Reference commit ce5b0921e0

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-ring-theory Ring theory label Dec 30, 2025
@vihdzp vihdzp requested a review from YaelDillies December 31, 2025 05:14
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 delegate

@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 31, 2025
@riccardobrasca
Copy link
Member

Thanks!

bors d+

@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Dec 31, 2025

✌️ vihdzp 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-mathlib4-bot leanprover-community-mathlib4-bot added delegated This pull request has been delegated to the PR author (or occasionally another non-maintainer). and removed maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. labels Dec 31, 2025
@vihdzp vihdzp added the awaiting-CI This PR doesn't pass CI yet. This label is automatically removed once it does. label Jan 2, 2026
@github-actions github-actions bot removed the awaiting-CI This PR doesn't pass CI yet. This label is automatically removed once it does. label Jan 2, 2026
@vihdzp
Copy link
Collaborator Author

vihdzp commented Jan 2, 2026

bors r+

mathlib-bors bot pushed a commit that referenced this pull request Jan 2, 2026
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jan 2, 2026

Pull request successfully merged into master.

Build succeeded!

And happy new year! 🎉

@mathlib-bors mathlib-bors bot changed the title feat: IsStrictOrderedRing (Lex R⟦Γ⟧) [Merged by Bors] - feat: IsStrictOrderedRing (Lex R⟦Γ⟧) Jan 2, 2026
@mathlib-bors mathlib-bors bot closed this Jan 2, 2026
kim-em pushed a commit to kim-em/mathlib4 that referenced this pull request Jan 6, 2026
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

delegated This pull request has been delegated to the PR author (or occasionally another non-maintainer). large-import Automatically added label for PRs with a significant increase in transitive imports t-ring-theory Ring theory

Projects

None yet

Development

Successfully merging this pull request may close these issues.

5 participants