Teichmüller lifts #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines witt_vector.teichmuller
, a monoid hom R →* 𝕎 R
, which embeds r : R
as the
0
-th component of a Witt vector whose other coefficients are 0
.
Main declarations #
witt_vector.teichmuller
: the Teichmuller map.witt_vector.map_teichmuller
:witt_vector.teichmuller
is a natural transformation.witt_vector.ghost_component_teichmuller
: then
-th ghost component ofwitt_vector.teichmuller p r
isr ^ p ^ n
.
References #
The underlying function of the monoid hom witt_vector.teichmuller
.
The 0
-th coefficient of teichmuller_fun p r
is r
, and all others are 0
.
teichmuller
is a monoid homomorphism #
On ghost components, it is clear that teichmuller_fun
is a monoid homomorphism.
But in general the ghost map is not injective.
We follow the same strategy as for proving that the ring operations on 𝕎 R
satisfy the ring axioms.
- We first prove it for rings
R
wherep
is invertible, because then the ghost map is in fact an isomorphism. - After that, we derive the result for
mv_polynomial R ℤ
, - and from that we can prove the result for arbitrary
R
.
The Teichmüller lift of an element of R
to 𝕎 R
.
The 0
-th coefficient of teichmuller p r
is r
, and all others are 0
.
This is a monoid homomorphism.
Equations
- witt_vector.teichmuller p = {to_fun := witt_vector.teichmuller_fun p _inst_1, map_one' := _, map_mul' := _}
teichmuller
is a natural transformation.
The n
-th ghost component of teichmuller p r
is r ^ p ^ n
.