mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(RingTheory/NoetherNormalization):Add noether normalization lemma

Open su00000 opened this issue 1 year ago • 2 comments

This PR contains a proof of Noether normalization lemma: Let A be a finitely generated algebra over a field k. Then there exists natural number $r$ and an injective homomorphism from k[X_1, X_2, ..., X_r] to A such that A is integral over k[X_1, X_2, ..., X_r].

Co-authored-by: Riccardo Brasca [email protected] Co-authored-by: Wan Lin [email protected] Co-authored-by: Xiaoyang Su [email protected]

  • [ ] depends on: #18244

Open in Gitpod

su00000 avatar Oct 26 '24 07:10 su00000

PR summary 613e535399

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.RingTheory.NoetherNormalization (new file) 1403

Declarations diff

+ Quotient.mk_bijective_iff_eq_bot + T1 + algebraMap_finiteType_iff_algebra_finiteType + exists_finite_inj_algHom_of_fg + exists_integral_inj_algHom_of_fg + exists_integral_inj_algHom_of_quotient + map_coe + ofDigits_inj_of_len_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).

github-actions[bot] avatar Oct 26 '24 07:10 github-actions[bot]

This PR/issue depends on:

  • ~~leanprover-community/mathlib4#18244~~ By Dependent Issues (🤖). Happy coding!

Can you please fix the conflict? Thanks!

riccardobrasca avatar Nov 15 '24 09:11 riccardobrasca

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

github-actions[bot] avatar Feb 18 '25 11:02 github-actions[bot]

Sorry, one last thing: can you add a TODO saying that we can take s in the final theorems equal to the Krull dimension of R?

riccardobrasca avatar Feb 18 '25 11:02 riccardobrasca

Sorry, one last thing: can you add a TODO saying that we can take s in the final theorems equal to the Krull dimension of R?

Sure

su00000 avatar Feb 18 '25 11:02 su00000

:v: su00000 can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

mathlib-bors[bot] avatar Feb 18 '25 11:02 mathlib-bors[bot]

bors r+

su00000 avatar Feb 18 '25 12:02 su00000

Build failed:

mathlib-bors[bot] avatar Feb 18 '25 12:02 mathlib-bors[bot]

Two hours without merging master and there is of course an error... it's probably a lemma about quotient that had implicitness of some variable changed. Feel free to fix and merge.

riccardobrasca avatar Feb 18 '25 12:02 riccardobrasca

I pushed a fix to Operations.lean but it will surely break something in the final file.

riccardobrasca avatar Feb 18 '25 13:02 riccardobrasca

bors r+

su00000 avatar Feb 18 '25 14:02 su00000

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Feb 18 '25 15:02 mathlib-bors[bot]