Witt vectors over a domain #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file builds to the proof witt_vector.is_domain
,
an instance that says if R
is an integral domain, then so is 𝕎 R
.
It depends on the API around iterated applications
of witt_vector.verschiebung
and witt_vector.frobenius
found in identities.lean
.
The proof sketch
goes as follows:
any nonzero $x$ is an iterated application of $V$
to some vector $w_x$ whose 0th component is nonzero (witt_vector.verschiebung_nonzero
).
Known identities (witt_vector.iterate_verschiebung_mul
) allow us to transform
the product of two such $x$ and $y$
to the form $V^{m+n}\left(F^n(w_x) \cdot F^m(w_y)\right)$,
the 0th component of which must be nonzero.
Main declarations #
witt_vector.iterate_verschiebung_mul_coeff
: an identity from [Haz09]witt_vector.is_domain
The shift
operator #
witt_vector.verschiebung
translates the entries of a Witt vector upward, inserting 0s in the gaps.
witt_vector.shift
does the opposite, removing the first entries.
This is mainly useful as an auxiliary construction for witt_vector.verschiebung_nonzero
.
Witt vectors over a domain #
If R
is an integral domain, then so is 𝕎 R
.
This argument is adapted from
https://math.stackexchange.com/questions/4117247/ring-of-witt-vectors-over-an-integral-domain/4118723#4118723.