Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

[Merged by Bors] - feat(number_theory): fundamental identity of ramification index and inertia degree #12287

Closed
wants to merge 6 commits into from

Conversation

Vierkantor
Copy link
Collaborator

@Vierkantor Vierkantor commented Feb 25, 2022

This PR proves the fundamental identity of ramification index and inertia degree:

Let p be a prime in a Dedekind domain R, S the integral closure of R in some finite field extension L of K = Frac(R), then for P ranging over the primes lying over p, Σ P, e P * f P = [L : K].


Open in Gitpod

@Vierkantor Vierkantor added the WIP Work in progress label Feb 25, 2022
Vierkantor added a commit that referenced this pull request Mar 2, 2022
bors bot pushed a commit that referenced this pull request Mar 3, 2022
@leanprover-community-bot-assistant leanprover-community-bot-assistant added the merge-conflict Please `git merge origin/master` then a bot will remove this label. label Apr 8, 2022
@leanprover-community-bot-assistant leanprover-community-bot-assistant added merge-conflict Please `git merge origin/master` then a bot will remove this label. and removed merge-conflict Please `git merge origin/master` then a bot will remove this label. labels Apr 11, 2022
@leanprover-community-bot-assistant leanprover-community-bot-assistant removed the merge-conflict Please `git merge origin/master` then a bot will remove this label. label May 2, 2022
@kim-em kim-em added the merge-conflict Please `git merge origin/master` then a bot will remove this label. label May 2, 2022
Vierkantor added a commit that referenced this pull request May 23, 2022
We define ramification index `ramification_idx` and inertia degree `inertia_deg` for `P : ideal S` over `p : ideal R` given a ring extension `f : R →+* S`. The literature generally assumes `p` is included in `P`, both are maximal, `R` is the ring of integers of a number field `K` and `S` is the integral closure of `R` in `L`, a finite separable extension of `K`; we relax these assumptions as much as is practical.

This PR was split off from #12287.
Vierkantor added a commit that referenced this pull request May 23, 2022
We define ramification index `ramification_idx` and inertia degree `inertia_deg` for `P : ideal S` over `p : ideal R` given a ring extension `f : R →+* S`. The literature generally assumes `p` is included in `P`, both are maximal, `R` is the ring of integers of a number field `K` and `S` is the integral closure of `R` in `L`, a finite separable extension of `K`; we relax these assumptions as much as is practical.

This PR was split off from #12287.
Vierkantor added a commit that referenced this pull request May 23, 2022
Two little lemmas on the set of factors which I needed for #12287.
bors bot pushed a commit that referenced this pull request May 23, 2022
…#14333)

Two little lemmas on the set of factors which I needed for #12287.



Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
@kbuzzard
Copy link
Member

It's really exciting that we're moving towards this; I have only just seen this PR! Thanks to Oliver for directing my attention towards it.

src/number_theory/ramification_inertia.lean Outdated Show resolved Hide resolved
/-- The **fundamental identity** of ramification index `e` and inertia degree `f`:
for `P` ranging over the primes lying over `p`, `∑ P, e P * f P = [Frac(S) : Frac(R)]`;
if `Frac(S) : Frac(R)` is a finite extension, `p` is maximal
and `S` is the integral closure of `R` in `L`. -/
Copy link
Member

Choose a reason for hiding this comment

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

As it stands this docstring isn't quite true (I was very confused by this for a minute or two!). The issue is that if Frac(S)/Frac(R) is finite then in this generality it's not enough to deduce that S is a Noetherian R-module. Here https://arxiv.org/abs/2102.10481 is a recent paper discussing a statement which is true in the generality of the docstring; however I am certainly suggesting we should be formalising it! The result proved is exactly what I need for several applications; all the applications to arithmetic have S a Noetherian (or equivalently finitely-generated, as R is Noetherian) R-module. For applications beyond arithmetic, I'm very happy to be worrying about them later :-) Note that S f.g. as R-module implies Frac(S) is finite over Frac(R).

Vierkantor added a commit that referenced this pull request Jul 13, 2022
(for a Dedekind domain `R` and its integral closure `S` and maximal ideal `p`)

This is the first step in showing the fundamental identity of inertia degree and ramification index (#12287).
The next step is to factor `pS` into coprime factors `P` and use the Chinese remainder theorem.
@Vierkantor Vierkantor added awaiting-review The author would like community review of the PR blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. and removed WIP Work in progress merge-conflict Please `git merge origin/master` then a bot will remove this label. labels Jul 13, 2022
@Vierkantor Vierkantor changed the title feat(number_theory): fundamental identity of ramification index and inertia degree [WIP] feat(number_theory): fundamental identity of ramification index and inertia degree Jul 13, 2022
bors bot pushed a commit that referenced this pull request Jul 19, 2022
#15315)

(for a Dedekind domain `R` and its integral closure `S` and maximal ideal `p`)

This is the first step in showing the fundamental identity of inertia degree and ramification index (#12287).
The next step is to factor `pS` into coprime factors `P` and use the Chinese remainder theorem.



Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
Co-authored-by: Anne Baanen <t.baanen@vu.nl>
joelriou pushed a commit that referenced this pull request Jul 23, 2022
#15315)

(for a Dedekind domain `R` and its integral closure `S` and maximal ideal `p`)

This is the first step in showing the fundamental identity of inertia degree and ramification index (#12287).
The next step is to factor `pS` into coprime factors `P` and use the Chinese remainder theorem.



Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
Co-authored-by: Anne Baanen <t.baanen@vu.nl>
bors bot pushed a commit that referenced this pull request Aug 4, 2022
…fication index (#15316)

Let `S` be a Dedekind domain extending the commutative ring `R`, `p` a maximal ideal of `R`, `P` a prime ideal of `S`, and `e` the (nonzero) ramification index of `P` over `p`. Because the ramification index is nonzero, we get an inclusion `R/p → S/P` and we can compute that the degree of the field extension `[S/(P^e) : R/p]` is exactly `e` times `[S/P : R/p]`.

This is the next step in showing the fundamental identity of inertia degree and ramification index (#12287).

Setting up the ingredients for the proof is quite complicated because it involves taking `(P^(i+1) / P^e)` as a `R/p`-subspace of `P^i / P^e` and basically each part of this structure would produce free metavariables if we naïvely assigned it an instance. In the end, the important parts are an instance for `S/(P^e)` as `R/p`-algebra and replacing subspaces with the image of inclusion maps.



Co-authored-by: Anne Baanen <t.baanen@vu.nl>
Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
@mathlib-dependent-issues-bot mathlib-dependent-issues-bot removed the blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. label Aug 4, 2022
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.

LGTM!

src/number_theory/ramification_inertia.lean Show resolved Hide resolved
Copy link
Member

@jcommelin jcommelin 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 merge

@leanprover-community-bot-assistant leanprover-community-bot-assistant added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Aug 17, 2022
bors bot pushed a commit that referenced this pull request Aug 17, 2022
…nertia degree (#12287)

This PR proves the fundamental identity of ramification index and inertia degree:

Let `p` be a prime in a Dedekind domain `R`, `S` the integral closure of `R` in some finite field extension `L` of `K = Frac(R)`, then for `P` ranging over the primes lying over `p`, `Σ P, e P * f P = [L : K]`.



Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
@bors
Copy link

bors bot commented Aug 17, 2022

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(number_theory): fundamental identity of ramification index and inertia degree [Merged by Bors] - feat(number_theory): fundamental identity of ramification index and inertia degree Aug 17, 2022
@bors bors bot closed this Aug 17, 2022
@bors bors bot deleted the ramification-inertia branch August 17, 2022 20:40
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

7 participants