mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(FieldTheory/Minpoly): minpoly K x splits implies minpoly K (algebraMap K L a - x) splits

Open jjdishere opened this issue 1 year ago • 6 comments

Add minpoly K x splits implies minpoly K (- x) splits and minpoly K (algebraMap K L a - x) splits. This is after #17093 .


  • [x] depends on: #17367
  • [ ] depends on: #17093 Open in Gitpod

jjdishere avatar Oct 02 '24 23:10 jjdishere

PR summary 8a41b52b74

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ Splits.comp_neg_X + Splits.comp_of_degree_le_one + Splits.comp_of_map_degree_le_one + algEquivAevalNegX + algEquivCMulXAddC + algEquivCMulXAddC_symm_eq + comp_neg_X_comp_neg_X + dvd_comp_C_mul_X_add_C_iff + dvd_comp_neg_X_iff + minpoly_algebraMap_sub_splits + minpoly_neg_splits + splits_iff_comp_splits_of_degree_eq_one

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 02 '24 23:10 github-actions[bot]

Doesn't IntermediateField.splits_of_mem_adjoin directly imply the result in the title (and #17903)?

alreadydone avatar Oct 08 '24 14:10 alreadydone

Doesn't IntermediateField.splits_of_mem_adjoin directly imply the result in the title (and #17903)?

Thank you very much @alreadydone ! I didn't find this theorem before. For those intermediate results in this PR, I believe they have their own use. For the final results, do you suggest I

  1. remove the final results, or
  2. keep them and use the IntermediateField.splits_of_mem_adjoin to golf the proof, or
  3. keep it as it is?

I think these final lemmas are easier to use than IntermediateField.splits_of_mem_adjoin in other proofs.

jjdishere avatar Oct 08 '24 15:10 jjdishere

~~Strangely the diff is still 34 files after you merged master~~ ... (I see, it's because #17403 is not yet merged) I'll take a look at the intermediate results after this is fixed. I think it's good to keep the final results and golf it, but if it requires additional import(s) you may keep your original proof.

alreadydone avatar Oct 08 '24 16:10 alreadydone

@alreadydone I've checked the dependency. IntermediateField.splits_of_mem_adjoin live in the file FieldTheory.Normal, which imports FieldTheory.SplittingField.Construction, which imports FieldTheory.SplittingField.IsSplittingField, which imports RingTheory.Adjoin.Field, which is the file my theorems live in.

So indeed it will require additional import(s) (move these lemmas to 3 files later) if I try to use IntermediateField.splits_of_mem_adjoin. What is your opinion on this?

jjdishere avatar Oct 08 '24 20:10 jjdishere

This PR/issue depends on:

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

maintainer merge

jcommelin avatar Nov 13 '24 14:11 jcommelin

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

github-actions[bot] avatar Nov 13 '24 14:11 github-actions[bot]

:v: jjdishere 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 Nov 13 '24 14:11 mathlib-bors[bot]

@jjdishere can you take into account the remaining comments and merge this (ignore the issue about {R} and {R : Type*} for now)? Thanks!

riccardobrasca avatar Nov 14 '24 10:11 riccardobrasca

bors r+

jjdishere avatar Nov 14 '24 17:11 jjdishere

Build failed:

mathlib-bors[bot] avatar Nov 14 '24 17:11 mathlib-bors[bot]

Can you please fix the error? Thanks!

riccardobrasca avatar Nov 18 '24 14:11 riccardobrasca

Can you please fix the error? Thanks!

Sorry for the delay! Fixed.

jjdishere avatar Nov 18 '24 19:11 jjdishere

bors r+

jjdishere avatar Nov 18 '24 19:11 jjdishere

Bors?

bors merge

riccardobrasca avatar Nov 19 '24 08:11 riccardobrasca

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Nov 19 '24 09:11 mathlib-bors[bot]