Pontryagin duality for finite abelian groups #
This file proves the Pontryagin duality in case of finite abelian groups. This states that any finite abelian group is canonically isomorphic to its double dual (the space of complex-valued characters of its space of complex-valued characters).
We first prove it for ZMod n
and then extend to all finite abelian groups using the
Structure Theorem.
TODO #
Reuse the work done in Mathlib.GroupTheory.FiniteAbelian.Duality
. This requires to write some more
glue.
Indexing of the complex characters of ZMod n
. AddChar.zmod n x
is the character sending y
to e ^ (2 * π * i * x * y / n)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
AddChar.zmod
bundled as an AddChar
.
Equations
- AddChar.zmodHom = { toFun := AddChar.zmod n, map_zero_eq_one' := ⋯, map_add_eq_mul' := ⋯ }
Instances For
The circle-valued characters of a finite abelian group are the same as its complex-valued characters.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Complex-valued characters of a finite abelian group α
form a basis of α → ℂ
.
Equations
Instances For
The double dual isomorphism of a finite abelian group.
Equations
- AddChar.doubleDualEquiv = AddEquiv.ofBijective AddChar.doubleDualEmb ⋯