Teichmüller lifts #
This file defines WittVector.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 #
WittVector.teichmuller
: the Teichmuller map.WittVector.map_teichmuller
:WittVector.teichmuller
is a natural transformation.WittVector.ghostComponent_teichmuller
: then
-th ghost component ofWittVector.teichmuller p r
isr ^ p ^ n
.
References #
The underlying function of the monoid hom WittVector.teichmuller
.
The 0
-th coefficient of teichmullerFun p r
is r
, and all others are 0
.
Equations
- WittVector.teichmullerFun p r = { coeff := fun (n : ℕ) => if n = 0 then r else 0 }
Instances For
teichmuller
is a monoid homomorphism #
On ghost components, it is clear that teichmullerFun
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
MvPolynomial 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
- WittVector.teichmuller p = { toFun := WittVector.teichmullerFun p, map_one' := ⋯, map_mul' := ⋯ }
Instances For
teichmuller
is a natural transformation.
The n
-th ghost component of teichmuller p r
is r ^ p ^ n
.