Documentation

Mathlib.RingTheory.DedekindDomain.SelmerGroup

Selmer groups of fraction fields of Dedekind domains #

Let $K$ be the field of fractions of a Dedekind domain $R$. For any set $S$ of prime ideals in the height one spectrum of $R$, and for any natural number $n$, the Selmer group $K(S, n)$ is defined to be the subgroup of the unit group $K^\times$ modulo $n$-th powers where each element has $v$-adic valuation divisible by $n$ for all prime ideals $v$ away from $S$. In other words, this is precisely $$ K(S, n) := {x(K^\times)^n \in K^\times / (K^\times)^n \ \mid

\forall v \notin S, \ \mathrm{ord}_v(x) \equiv 0 \pmod n}. $$

There is a fundamental short exact sequence $$ 1 \to R_S^\times / (R_S^\times)^n \to K(S, n) \to \mathrm{Cl}_S(R)[n] \to 0, $$ where $R_S^\times$ is the $S$-unit group of $R$ and $\mathrm{Cl}_S(R)$ is the $S$-class group of $R$. If the flanking groups are both finite, then $K(S, n)$ is finite by the first isomorphism theorem. Such is the case when $R$ is the ring of integers of a number field $K$, $S$ is finite, and $n$ is positive, in which case $R_S^\times$ is finitely generated by Dirichlet's unit theorem and $\mathrm{Cl}_S(R)$ is finite by the class number theorem.

This file defines the Selmer group $K(S, n)$ and some basic facts.

Main definitions #

Main statements #

Notations #

Implementation notes #

The Selmer group is typically defined as a subgroup of the Galois cohomology group $H^1(K, \mu_n)$ with certain local conditions defined by $v$-adic valuations, where $\mu_n$ is the group of $n$-th roots of unity over a separable closure of $K$. Here $H^1(K, \mu_n)$ is identified with $K^\times / (K^\times)^n$ by the long exact sequence from Kummer theory and Hilbert's theorem 90, and the fundamental short exact sequence becomes an easy consequence of the snake lemma. This file will define all the maps explicitly for computational purposes, but isomorphisms to the Galois cohomological definition will be provided when possible.

References #

https://doc.sagemath.org/html/en/reference/number_fields/sage/rings/number_field/selmer_group.html

Tags #

class group, selmer group, unit group

Valuations of non-zero elements #

The multiplicative v-adic valuation on .

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    The multiplicative v-adic valuation on .

    Equations
    Instances For

      The multiplicative v-adic valuation on modulo n-th powers.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        Selmer groups #

        The Selmer group K⟮S, n⟯.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem IsDedekindDomain.selmerGroup.monotone {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {S : Set (IsDedekindDomain.HeightOneSpectrum R)} {S' : Set (IsDedekindDomain.HeightOneSpectrum R)} {n : } (hS : S S') :
          IsDedekindDomain.selmerGroup IsDedekindDomain.selmerGroup
          def IsDedekindDomain.selmerGroup.valuation {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {S : Set (IsDedekindDomain.HeightOneSpectrum R)} {n : } :
          IsDedekindDomain.selmerGroup →* SMultiplicative (ZMod n)

          The multiplicative v-adic valuations on K⟮S, n⟯ for all v ∈ S.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem IsDedekindDomain.selmerGroup.valuation_ker_eq {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {S : Set (IsDedekindDomain.HeightOneSpectrum R)} {n : } :
            MonoidHom.ker IsDedekindDomain.selmerGroup.valuation = Subgroup.subgroupOf IsDedekindDomain.selmerGroup IsDedekindDomain.selmerGroup
            def IsDedekindDomain.selmerGroup.fromUnit {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {n : } :
            Rˣ →* IsDedekindDomain.selmerGroup

            The natural homomorphism from to K⟮∅, n⟯.

            Equations
            • IsDedekindDomain.selmerGroup.fromUnit = { toOneHom := { toFun := fun (x : Rˣ) => { val := ((Units.map (algebraMap R K)) x), property := }, map_one' := }, map_mul' := }
            Instances For
              theorem IsDedekindDomain.selmerGroup.fromUnit_ker {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {n : } [hn : Fact (0 < n)] :
              MonoidHom.ker IsDedekindDomain.selmerGroup.fromUnit = MonoidHom.range (powMonoidHom n)
              def IsDedekindDomain.selmerGroup.fromUnitLift {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {n : } [Fact (0 < n)] :
              Rˣ MonoidHom.range (powMonoidHom n) →* IsDedekindDomain.selmerGroup

              The injection induced by the natural homomorphism from to K⟮∅, n⟯.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                theorem IsDedekindDomain.selmerGroup.fromUnitLift_injective {R : Type u} [CommRing R] [IsDedekindDomain R] {K : Type v} [Field K] [Algebra R K] [IsFractionRing R K] {n : } [Fact (0 < n)] :
                Function.Injective IsDedekindDomain.selmerGroup.fromUnitLift