Documentation

Mathlib.RingTheory.DedekindDomain.FiniteAdeleRing

The finite adèle ring of a Dedekind domain #

We define the ring of finite adèles of a Dedekind domain R.

Main definitions #

Implementation notes #

We are only interested on Dedekind domains of Krull dimension 1 (i.e., not fields). If R is a field, its finite adèle ring is just defined to be the trivial ring.

References #

Tags #

finite adèle ring, dedekind domain

def DedekindDomain.FiniteIntegralAdeles (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] :
Type (max u_1 u_2)

The product of all adicCompletionIntegers, where v runs over the maximal ideals of R.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def DedekindDomain.ProdAdicCompletions (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] :
          Type (max u_1 u_2)

          The product of all adicCompletion, where v runs over the maximal ideals of R.

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

                The inclusion of R_hat in K_hat as a homomorphism of additive monoids.

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

                  The inclusion of R_hat in K_hat as a ring homomorphism.

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

                    The inclusion of R_hat in K_hat as an algebra homomorphism.

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

                      The finite adèle ring of a Dedekind domain #

                      We define the finite adèle ring of R as the restricted product over all maximal ideals v of R of adicCompletion with respect to adicCompletionIntegers. We prove that it is a commutative ring.

                      An element x : K_hat R K is a finite adèle if for all but finitely many height one ideals v, the component x v is a v-adic integer.

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

                        The sum of two finite adèles is a finite adèle.

                        The tuple (0)_v is a finite adèle.

                        The negative of a finite adèle is a finite adèle.

                        The product of two finite adèles is a finite adèle.

                        The tuple (1)_v is a finite adèle.

                        def DedekindDomain.FiniteAdeleRing (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] :
                        Type (max u_1 u_2)

                        The finite adèle ring of R is the restricted product over all maximal ideals v of R of adicCompletion, with respect to adicCompletionIntegers.

                        Note that we make this a Type rather than a Subtype (e.g., a Subalgebra) since we wish to endow it with a finer topology than that of the subspace topology.

                        Equations
                        Instances For

                          The finite adèle ring of R, regarded as a K-subalgebra of the product of the local completions of K.

                          Note that this definition exists to streamline the proof that the finite adèles are an algebra over K, rather than to express their relationship to K_hat R K which is essentially a detail of their construction.

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            theorem DedekindDomain.FiniteAdeleRing.ext (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] {a₁ a₂ : FiniteAdeleRing R K} (h : Eq a₁.val a₂.val) :
                            Eq a₁ a₂
                            theorem DedekindDomain.FiniteAdeleRing.ext_iff {R : Type u_1} {K : Type u_2} [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] {a₁ a₂ : FiniteAdeleRing R K} :
                            Iff (Eq a₁ a₂) (Eq a₁.val a₂.val)

                            The finite adele ring is an algebra over the finite integral adeles.

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