Skip to content

Conversation

acmepjz
Copy link
Collaborator

@acmepjz acmepjz commented Jun 26, 2025

Proved IsCyclotomicExtension.isMulCommutative that any cyclotomic extension (of rings) is abelian.

Deprecated IsCyclotomicExtension.Aut.commGroup which is CommGroup and only adjoins one root of unity. Now CommGroup instance should be inferred automatically if IsMulCommutative is provided (the preferred spelling of abelian extension, see #23669 (comment)).


Open in Gitpod

@acmepjz acmepjz added t-algebra Algebra (groups, rings, fields, etc) awaiting-CI This PR doesn't pass CI yet. This label is automatically removed once it does. labels Jun 26, 2025
@acmepjz acmepjz changed the title feat(): any cyclotomic extension is abelian feat(NumberTheory/Cyclotomic/Basic): any cyclotomic extension is abelian Jun 26, 2025
@github-actions github-actions bot added the t-number-theory Number theory (also use t-algebra or t-analysis to specialize) label Jun 26, 2025
Copy link

github-actions bot commented Jun 26, 2025

PR summary c873c5d1d1

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ algEquiv_eq_of_apply_eq
+ isMulCommutative

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

@acmepjz acmepjz added the WIP Work in progress label Jun 26, 2025
@acmepjz acmepjz removed the WIP Work in progress label Jun 26, 2025
@acmepjz
Copy link
Collaborator Author

acmepjz commented Jun 26, 2025

What's wrong with Post-Build Step (fork)?

@mbkybky
Copy link
Collaborator

mbkybky commented Jun 26, 2025

What's wrong with Post-Build Step (fork)?

See zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Failing.20CI

@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 Jun 27, 2025
@riccardobrasca riccardobrasca self-assigned this Jun 29, 2025
@acmepjz acmepjz requested a review from riccardobrasca June 29, 2025 11:23
Copy link
Member

@riccardobrasca riccardobrasca left a comment

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Thanks!

bors d+

@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jun 30, 2025

✌️ acmepjz 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 the delegated This pull request has been delegated to the PR author (or occasionally another non-maintainer). label Jun 30, 2025
Co-authored-by: Riccardo Brasca <riccardo.brasca@gmail.com>
@acmepjz
Copy link
Collaborator Author

acmepjz commented Jun 30, 2025

bors r+

mathlib-bors bot pushed a commit that referenced this pull request Jun 30, 2025
…ian (#26427)

Proved `IsCyclotomicExtension.isMulCommutative` that any cyclotomic extension (of rings) is abelian.

Deprecated `IsCyclotomicExtension.Aut.commGroup` which is `CommGroup` and only adjoins one root of unity. Now `CommGroup` instance should be inferred automatically if `IsMulCommutative` is provided (the preferred spelling of abelian extension, see #23669 (comment)).
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jun 30, 2025

This PR was included in a batch that successfully built, but then failed to merge into master (it was a non-fast-forward update). It will be automatically retried.

mathlib-bors bot pushed a commit that referenced this pull request Jun 30, 2025
…ian (#26427)

Proved `IsCyclotomicExtension.isMulCommutative` that any cyclotomic extension (of rings) is abelian.

Deprecated `IsCyclotomicExtension.Aut.commGroup` which is `CommGroup` and only adjoins one root of unity. Now `CommGroup` instance should be inferred automatically if `IsMulCommutative` is provided (the preferred spelling of abelian extension, see #23669 (comment)).
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Jun 30, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feat(NumberTheory/Cyclotomic/Basic): any cyclotomic extension is abelian [Merged by Bors] - feat(NumberTheory/Cyclotomic/Basic): any cyclotomic extension is abelian Jun 30, 2025
@mathlib-bors mathlib-bors bot closed this Jun 30, 2025
@acmepjz acmepjz deleted the acmepjz_cyc_abelian branch June 30, 2025 14:18
joelriou pushed a commit to joelriou/mathlib4 that referenced this pull request Jul 7, 2025
…ian (leanprover-community#26427)

Proved `IsCyclotomicExtension.isMulCommutative` that any cyclotomic extension (of rings) is abelian.

Deprecated `IsCyclotomicExtension.Aut.commGroup` which is `CommGroup` and only adjoins one root of unity. Now `CommGroup` instance should be inferred automatically if `IsMulCommutative` is provided (the preferred spelling of abelian extension, see leanprover-community#23669 (comment)).
callesonne pushed a commit to callesonne/mathlib4 that referenced this pull request Jul 24, 2025
…ian (leanprover-community#26427)

Proved `IsCyclotomicExtension.isMulCommutative` that any cyclotomic extension (of rings) is abelian.

Deprecated `IsCyclotomicExtension.Aut.commGroup` which is `CommGroup` and only adjoins one root of unity. Now `CommGroup` instance should be inferred automatically if `IsMulCommutative` is provided (the preferred spelling of abelian extension, see leanprover-community#23669 (comment)).
hrmacbeth pushed a commit to szqzs/mathlib4 that referenced this pull request Jul 28, 2025
…ian (leanprover-community#26427)

Proved `IsCyclotomicExtension.isMulCommutative` that any cyclotomic extension (of rings) is abelian.

Deprecated `IsCyclotomicExtension.Aut.commGroup` which is `CommGroup` and only adjoins one root of unity. Now `CommGroup` instance should be inferred automatically if `IsMulCommutative` is provided (the preferred spelling of abelian extension, see leanprover-community#23669 (comment)).
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). t-algebra Algebra (groups, rings, fields, etc) t-number-theory Number theory (also use t-algebra or t-analysis to specialize)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

4 participants