Skip to content

Conversation

@BoltonBailey
Copy link
Collaborator

@BoltonBailey BoltonBailey commented Jun 15, 2025

This PR creates a new file for lemmas about MvPolynomials over rings which are NoZeroDivisors, to make modified versions of lemmas like degreeOf_C_mul.

Original PR: #11106


Notes to self:

  • Can the results in this file be generalized?
  • Perhaps to the assumption IsCancelMulZero R?
    • Note that when R is a ring, IsCancelMulZero R is equivalent to
      NoZeroDivisors R.
    • When R is only a semiring, NoZeroDivisors R is implied by IsCancelMulZero R
      (although this is not typeclass inferrable, see IsLeftCancelMulZero.to_noZeroDivisors),
    • When R is only a semiring, IsCancelMulZero R is not implied by NoZeroDivisors R, see https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/IsCancelMulZero.20and.20NoZeroDivisors.20for.20semirings/with/562333254
    • Thus, we should see if the results in this file can be generalized to
      IsCancelMulZero R.
    • Note that MvPolynomial.totalDegree_mul_of_isDomain exists, which proves a related result
      under the assumption IsCancelMulZero R.
    • This seems weaker than it could be!
    • I will try to open PR to generalize these results to NoZeroDivisors R in a new PR.
  • Perhaps to more specific assumptions about cancellation on leadingCoeffs?

This PR continues the work from #11106 and #11073

@github-actions github-actions bot added the t-algebra Algebra (groups, rings, fields, etc) label Jun 15, 2025
@github-actions
Copy link

github-actions bot commented Jun 15, 2025

PR summary 519f4546a1

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.FieldTheory.SeparablyGenerated Mathlib.RingTheory.MvPolynomial.IrreducibleQuadratic 1
Mathlib.Algebra.MvPolynomial.NoZeroDivisors (new file) 1028

Declarations diff

+ degreeOf_C_mul
+ degreeOf_mul_eq
+ degreeOf_one
+ degreeOf_pow_eq
+ degreeOf_prod_eq
+ degrees_mul_eq

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

@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot added the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Jun 21, 2025
@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot removed the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Dec 4, 2025
@BoltonBailey BoltonBailey marked this pull request as ready for review December 6, 2025 01:01
@erdOne erdOne added the awaiting-author A reviewer has asked the author a question or requested changes. label Dec 6, 2025
BoltonBailey and others added 2 commits December 6, 2025 16:23
Co-authored-by: Andrew Yang <36414270+erdOne@users.noreply.github.com>
@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot added blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) and removed blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) labels Dec 7, 2025
@BoltonBailey BoltonBailey added the awaiting-CI This PR doesn't pass CI yet. This label is automatically removed once it does. label Dec 30, 2025
@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 Dec 30, 2025
BoltonBailey and others added 8 commits January 1, 2026 20:47
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
…:BoltonBailey/mathlib4 into BoltonBailey/MvPolynomial.NoZeroDivisors
BoltonBailey and others added 9 commits January 2, 2026 11:55
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
@riccardobrasca
Copy link
Member

I think we can live with aesop instead of grind at the moment, so this LGTM, thanks!

bors merge

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the ready-to-merge This PR has been sent to bors. label Jan 3, 2026
mathlib-bors bot pushed a commit that referenced this pull request Jan 3, 2026
This PR creates a new file for lemmas about `MvPolynomial`s over rings which are `NoZeroDivisors`, to make modified versions of lemmas like `degreeOf_C_mul`.

Original PR: #11106

- [x] depends on: #11095
- [x] depends on: #11094
- [x] depends on: #25926 [We need this lemma to establish fact about degreeOf n (p + q)]
- [x] depends on: #32558
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jan 3, 2026

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feat: file for lemmas about MvPolynomials over NoZeroDivisors [Merged by Bors] - feat: file for lemmas about MvPolynomials over NoZeroDivisors Jan 3, 2026
@mathlib-bors mathlib-bors bot closed this Jan 3, 2026
kim-em pushed a commit to kim-em/mathlib4 that referenced this pull request Jan 6, 2026
…over-community#25925)

This PR creates a new file for lemmas about `MvPolynomial`s over rings which are `NoZeroDivisors`, to make modified versions of lemmas like `degreeOf_C_mul`.

Original PR: leanprover-community#11106

- [x] depends on: leanprover-community#11095
- [x] depends on: leanprover-community#11094
- [x] depends on: leanprover-community#25926 [We need this lemma to establish fact about degreeOf n (p + q)]
- [x] depends on: leanprover-community#32558
@adomani adomani mentioned this pull request Jan 16, 2026
goliath-klein pushed a commit to PrParadoxy/mathlib4 that referenced this pull request Jan 24, 2026
…over-community#25925)

This PR creates a new file for lemmas about `MvPolynomial`s over rings which are `NoZeroDivisors`, to make modified versions of lemmas like `degreeOf_C_mul`.

Original PR: leanprover-community#11106

- [x] depends on: leanprover-community#11095
- [x] depends on: leanprover-community#11094
- [x] depends on: leanprover-community#25926 [We need this lemma to establish fact about degreeOf n (p + q)]
- [x] depends on: leanprover-community#32558
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