Documentation

Mathlib.RingTheory.WittVector.WittPolynomial

Witt polynomials #

To endow WittVector p R with a ring structure, we need to study the so-called Witt polynomials.

Fix a base value p : ℕ. The p-adic Witt polynomials are an infinite family of polynomials indexed by a natural number n, taking values in an arbitrary ring R. The variables of these polynomials are represented by natural numbers. The variable set of the nth Witt polynomial contains at most n+1 elements {0, ..., n}, with exactly these variables when R has characteristic 0.

These polynomials are used to define the addition and multiplication operators on the type of Witt vectors. (While this type itself is not complicated, the ring operations are what make it interesting.)

When the base p is invertible in R, the p-adic Witt polynomials form a basis for MvPolynomial ℕ R, equivalent to the standard basis.

Main declarations #

Notation #

In this file we use the following notation

References #

noncomputable def wittPolynomial (p : ) (R : Type u_1) [CommRing R] (n : ) :

wittPolynomial p R n is the n-th Witt polynomial with respect to a prime p with coefficients in a commutative ring R. It is defined as:

∑_{i ≤ n} p^i X_i^{p^{n-i}} ∈ R[X_0, X_1, X_2, …].

Equations
Instances For
    theorem wittPolynomial_eq_sum_C_mul_X_pow (p : ) (R : Type u_1) [CommRing R] (n : ) :
    wittPolynomial p R n = Finset.sum (Finset.range (n + 1)) fun (i : ) => MvPolynomial.C (p ^ i) * MvPolynomial.X i ^ p ^ (n - i)

    We set up notation locally to this file, to keep statements short and comprehensible. This allows us to simply write W n or W_ ℤ n.

    wittPolynomial p R n is the n-th Witt polynomial with respect to a prime p with coefficients in a commutative ring R. It is defined as:

    ∑_{i ≤ n} p^i X_i^{p^{n-i}} ∈ R[X_0, X_1, X_2, …].

    Equations
    Instances For

      wittPolynomial p R n is the n-th Witt polynomial with respect to a prime p with coefficients in a commutative ring R. It is defined as:

      ∑_{i ≤ n} p^i X_i^{p^{n-i}} ∈ R[X_0, X_1, X_2, …].

      Equations
      Instances For

        The first observation is that the Witt polynomial doesn't really depend on the coefficient ring. If we map the coefficients through a ring homomorphism, we obtain the corresponding Witt polynomial over the target ring.

        @[simp]
        theorem map_wittPolynomial (p : ) {R : Type u_1} [CommRing R] {S : Type u_2} [CommRing S] (f : R →+* S) (n : ) :
        @[simp]
        theorem constantCoeff_wittPolynomial (p : ) (R : Type u_1) [CommRing R] [hp : Fact (Nat.Prime p)] (n : ) :
        MvPolynomial.constantCoeff (wittPolynomial p R n) = 0
        @[simp]
        theorem wittPolynomial_zero (p : ) (R : Type u_1) [CommRing R] :
        @[simp]
        theorem wittPolynomial_one (p : ) (R : Type u_1) [CommRing R] :
        wittPolynomial p R 1 = MvPolynomial.C p * MvPolynomial.X 1 + MvPolynomial.X 0 ^ p
        theorem aeval_wittPolynomial (p : ) (R : Type u_1) [CommRing R] {A : Type u_3} [CommRing A] [Algebra R A] (f : A) (n : ) :
        (MvPolynomial.aeval f) (wittPolynomial p R n) = Finset.sum (Finset.range (n + 1)) fun (i : ) => p ^ i * f i ^ p ^ (n - i)
        @[simp]
        theorem wittPolynomial_zmod_self (p : ) (n : ) :
        wittPolynomial p (ZMod (p ^ (n + 1))) (n + 1) = (MvPolynomial.expand p) (wittPolynomial p (ZMod (p ^ (n + 1))) n)

        Over the ring ZMod (p^(n+1)), we produce the n+1st Witt polynomial by expanding the nth Witt polynomial by p.

        theorem wittPolynomial_vars (p : ) (R : Type u_1) [CommRing R] [hp : NeZero p] [CharZero R] (n : ) :

        Witt polynomials as a basis of the polynomial algebra #

        If p is invertible in R, then the Witt polynomials form a basis of the polynomial algebra MvPolynomial ℕ R. The polynomials xInTermsOfW give the coordinate transformation in the backwards direction.

        noncomputable def xInTermsOfW (p : ) (R : Type u_1) [CommRing R] [Invertible p] :

        The xInTermsOfW p R n is the polynomial on the basis of Witt polynomials that corresponds to the ordinary X n.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem xInTermsOfW_eq (p : ) (R : Type u_1) [CommRing R] [Invertible p] {n : } :
          xInTermsOfW p R n = (MvPolynomial.X n - Finset.sum (Finset.range n) fun (i : ) => MvPolynomial.C (p ^ i) * xInTermsOfW p R i ^ p ^ (n - i)) * MvPolynomial.C (p ^ n)
          @[simp]
          theorem constantCoeff_xInTermsOfW (p : ) (R : Type u_1) [CommRing R] [hp : Fact (Nat.Prime p)] [Invertible p] (n : ) :
          MvPolynomial.constantCoeff (xInTermsOfW p R n) = 0
          @[simp]
          theorem xInTermsOfW_zero (p : ) (R : Type u_1) [CommRing R] [Invertible p] :
          theorem xInTermsOfW_aux (p : ) (R : Type u_1) [CommRing R] [Invertible p] (n : ) :
          xInTermsOfW p R n * MvPolynomial.C (p ^ n) = MvPolynomial.X n - Finset.sum (Finset.range n) fun (i : ) => MvPolynomial.C (p ^ i) * xInTermsOfW p R i ^ p ^ (n - i)