Skip to content

Conversation

@mans0954
Copy link
Collaborator

@mans0954 mans0954 commented May 21, 2024

Refactor Algebra.Star.Order to use the new non-unital *-ring homomorphisms / isomorphisms introduced in #12924


Open in Gitpod

mans0954 and others added 27 commits May 15, 2024 06:14
@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label May 21, 2024
@github-actions
Copy link

github-actions bot commented Jun 7, 2024

Import summary

No significant changes to the import graph

@github-actions
Copy link

github-actions bot commented Jun 15, 2024

PR summary 809384e3dd

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.Algebra.Star.Order 507 508 +1 (+0.20%)
Import changes for all files
Files Import difference
24 files Mathlib.Analysis.SpecialFunctions.Trigonometric.Chebyshev Mathlib.Analysis.Calculus.FDeriv.Analytic Mathlib.Data.Complex.Exponential Mathlib.Algebra.Order.Ring.Star Mathlib.LinearAlgebra.Matrix.DotProduct Mathlib.Data.Matrix.Rank Mathlib.Data.Rat.Star Mathlib.Algebra.Star.CHSH Mathlib.Algebra.Star.Order Mathlib.Data.Int.Star Mathlib.Analysis.Analytic.Meromorphic Mathlib.Analysis.Calculus.LocalExtr.Polynomial Mathlib.Data.Real.StarOrdered Mathlib.Analysis.Analytic.Linear Mathlib.Analysis.Analytic.Constructions Mathlib.Analysis.Analytic.Composition Mathlib.Analysis.Analytic.Basic Mathlib.Analysis.Analytic.Uniqueness Mathlib.Analysis.Analytic.CPolynomial Mathlib.Geometry.Manifold.AnalyticManifold Mathlib.LinearAlgebra.Matrix.GeneralLinearGroup.Card Mathlib.Analysis.Analytic.IsolatedZeros Mathlib.Analysis.Analytic.Inverse Mathlib.Analysis.Analytic.Polynomial
1

Declarations diff

+ NonUnitalStarRingHom.map_le_map_of_map_star
+ instance (priority := 100) StarRingEquivClass.instOrderIsoClass [EquivLike F R S]
+ instance (priority := 100) StarRingHomClass.instOrderHomClass [FunLike F R S]
- NonUnitalRingHom.map_le_map_of_map_star
- instance (priority := 100) StarRingHomClass.instOrderHomClass [FunLike F R S] [StarHomClass F R S]
- instance (priority := 100) StarRingHomClass.instOrderIsoClass [EquivLike F R S] [StarHomClass F R 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>

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-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 Jun 17, 2024
@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot removed merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) labels Jun 23, 2024
@leanprover-community-mathlib4-bot
Copy link
Collaborator

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-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 Jun 26, 2024
@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot removed the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Jun 27, 2024
@riccardobrasca riccardobrasca added the WIP Work in progress label Jul 5, 2024
@mans0954 mans0954 removed the WIP Work in progress label Jul 13, 2024
@mans0954
Copy link
Collaborator Author

mans0954 commented Jul 13, 2024

@riccardobrasca I assume you added the WIP label because I previously forgot to tag this with the now-defunct awaiting-review label rather than because you thought some further work was needed?

@riccardobrasca
Copy link
Member

@riccardobrasca I assume you added the WIP label because I previously forgot to tag this with the now-defunct awaiting-review label rather than because you thought some further work was needed?

Yes, feel free to remove it if it's ready for reviews.

@mans0954 mans0954 added the t-algebra Algebra (groups, rings, fields, etc) label Jul 14, 2024
@kim-em
Copy link
Contributor

kim-em commented Jul 15, 2024

bors merge

@github-actions github-actions bot added the ready-to-merge This PR has been sent to bors. label Jul 15, 2024
mathlib-bors bot pushed a commit that referenced this pull request Jul 15, 2024
…r.Order (#13089)

Refactor `Algebra.Star.Order` to use the new non-unital *-ring homomorphisms / isomorphisms introduced in #12924



Co-authored-by: Christopher Hoskin <[email protected]>
Co-authored-by: Christopher Hoskin <[email protected]>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jul 15, 2024

Build failed (retrying...):

mathlib-bors bot pushed a commit that referenced this pull request Jul 16, 2024
…r.Order (#13089)

Refactor `Algebra.Star.Order` to use the new non-unital *-ring homomorphisms / isomorphisms introduced in #12924



Co-authored-by: Christopher Hoskin <[email protected]>
Co-authored-by: Christopher Hoskin <[email protected]>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jul 16, 2024

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title refactor(Algebra/Star/Order): Use NonUnitalStarRingHom in Algebra.Star.Order [Merged by Bors] - refactor(Algebra/Star/Order): Use NonUnitalStarRingHom in Algebra.Star.Order Jul 16, 2024
@mathlib-bors mathlib-bors bot closed this Jul 16, 2024
@mathlib-bors mathlib-bors bot deleted the mans0954/StarRingEquivClass.instOrderIsoClass branch July 16, 2024 01:36
@adomani adomani mentioned this pull request Aug 1, 2024
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.

6 participants