mathlib3 documentation

ring_theory.witt_vector.defs

Witt vectors #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we define the type of p-typical Witt vectors and ring operations on it. The ring axioms are verified in ring_theory/witt_vector/basic.lean.

For a fixed commutative ring R and prime p, a Witt vector x : 𝕎 R is an infinite sequence ℕ → R of elements of R. However, the ring operations + and * are not defined in the obvious component-wise way. Instead, these operations are defined via certain polynomials using the machinery in structure_polynomial.lean. The nth value of the sum of two Witt vectors can depend on the 0-th through nth values of the summands. This effectively simulates a “carrying” operation.

Main definitions #

Notation #

We use notation 𝕎 R, entered \bbW, for the Witt vectors over R.

References #

structure witt_vector (p : ) (R : Type u_1) :
Type u_1

witt_vector p R is the ring of p-typical Witt vectors over the commutative ring R, where p is a prime number.

If p is invertible in R, this ring is isomorphic to ℕ → R (the product of copies of R). If R is a ring of characteristic p, then witt_vector p R is a ring of characteristic 0. The canonical example is witt_vector p (zmod p), which is isomorphic to the p-adic integers ℤ_[p].

Instances for witt_vector
@[ext]
theorem witt_vector.ext {p : } {R : Type u_1} {x y : witt_vector p R} (h : (n : ), x.coeff n = y.coeff n) :
x = y
theorem witt_vector.ext_iff {p : } {R : Type u_1} {x y : witt_vector p R} :
x = y (n : ), x.coeff n = y.coeff n
theorem witt_vector.coeff_mk (p : ) {R : Type u_1} (x : R) :
{coeff := x}.coeff = x
@[protected, instance]
Equations
@[protected, instance]
noncomputable def witt_vector.witt_zero (p : ) [hp : fact (nat.prime p)] :

The polynomials used for defining the element 0 of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_one (p : ) [hp : fact (nat.prime p)] :

The polynomials used for defining the element 1 of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_add (p : ) [hp : fact (nat.prime p)] :

The polynomials used for defining the addition of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_nsmul (p : ) [hp : fact (nat.prime p)] (n : ) :

The polynomials used for defining repeated addition of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_zsmul (p : ) [hp : fact (nat.prime p)] (n : ) :

The polynomials used for defining repeated addition of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_sub (p : ) [hp : fact (nat.prime p)] :

The polynomials used for describing the subtraction of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_mul (p : ) [hp : fact (nat.prime p)] :

The polynomials used for defining the multiplication of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_neg (p : ) [hp : fact (nat.prime p)] :

The polynomials used for defining the negation of the ring of Witt vectors.

Equations
noncomputable def witt_vector.witt_pow (p : ) [hp : fact (nat.prime p)] (n : ) :

The polynomials used for defining repeated addition of the ring of Witt vectors.

Equations
noncomputable def witt_vector.peval {R : Type u_1} [comm_ring R] {k : } (φ : mv_polynomial (fin k × ) ) (x : fin k R) :
R

An auxiliary definition used in witt_vector.eval. Evaluates a polynomial whose variables come from the disjoint union of k copies of , with a curried evaluation x. This can be defined more generally but we use only a specific instance here.

Equations
noncomputable def witt_vector.eval {p : } {R : Type u_1} [comm_ring R] {k : } (φ : mv_polynomial (fin k × ) ) (x : fin k witt_vector p R) :

Let φ be a family of polynomials, indexed by natural numbers, whose variables come from the disjoint union of k copies of , and let xᵢ be a Witt vector for 0 ≤ i < k.

eval φ x evaluates φ mapping the variable X_(i, n) to the nth coefficient of xᵢ.

Instantiating φ with certain polynomials defined in structure_polynomial.lean establishes the ring operations on 𝕎 R. For example, witt_vector.witt_add is such a φ with k = 2; evaluating this at (x₀, x₁) gives us the sum of two Witt vectors x₀ + x₁.

Equations
@[protected, instance]
noncomputable def witt_vector.has_zero {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.inhabited {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_one {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_add {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_sub {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_nat_scalar {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_int_scalar {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_mul {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_neg {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_nat_pow {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_nat_cast {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[protected, instance]
noncomputable def witt_vector.has_int_cast {p : } (R : Type u_1) [comm_ring R] [fact (nat.prime p)] :
Equations
@[simp]
theorem witt_vector.witt_zero_eq_zero (p : ) [hp : fact (nat.prime p)] (n : ) :
@[simp]
@[simp]
theorem witt_vector.witt_one_pos_eq_zero (p : ) [hp : fact (nat.prime p)] (n : ) (hn : 0 < n) :
@[simp]
@[simp]
theorem witt_vector.zero_coeff (p : ) (R : Type u_1) [hp : fact (nat.prime p)] [comm_ring R] (n : ) :
0.coeff n = 0
@[simp]
theorem witt_vector.one_coeff_zero (p : ) (R : Type u_1) [hp : fact (nat.prime p)] [comm_ring R] :
1.coeff 0 = 1
@[simp]
theorem witt_vector.one_coeff_eq_of_pos (p : ) (R : Type u_1) [hp : fact (nat.prime p)] [comm_ring R] (n : ) (hn : 0 < n) :
1.coeff n = 0
@[simp]
theorem witt_vector.v2_coeff {p' : } {R' : Type u_1} (x y : witt_vector p' R') (i : fin 2) :
(![x, y] i).coeff = ![x.coeff, y.coeff] i
theorem witt_vector.add_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x y : witt_vector p R) (n : ) :
theorem witt_vector.sub_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x y : witt_vector p R) (n : ) :
theorem witt_vector.mul_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x y : witt_vector p R) (n : ) :
theorem witt_vector.neg_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x : witt_vector p R) (n : ) :
theorem witt_vector.nsmul_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (m : ) (x : witt_vector p R) (n : ) :
theorem witt_vector.zsmul_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (m : ) (x : witt_vector p R) (n : ) :
theorem witt_vector.pow_coeff {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (m : ) (x : witt_vector p R) (n : ) :
theorem witt_vector.add_coeff_zero {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x y : witt_vector p R) :
(x + y).coeff 0 = x.coeff 0 + y.coeff 0
theorem witt_vector.mul_coeff_zero {p : } {R : Type u_1} [hp : fact (nat.prime p)] [comm_ring R] (x y : witt_vector p R) :
(x * y).coeff 0 = x.coeff 0 * y.coeff 0