q-expansions of modular forms #
We show that a modular form of level Ξ(n)
can be written as Ο β¦ F (π’ n Ο)
where F
is
analytic on the open unit disc, and π’ n
is the parameter Ο β¦ exp (2 * I * Ο * Ο / n)
. As an
application, we show that cusp forms decay exponentially to 0 as im Ο β β
.
TO DO: #
- generalise to handle arbitrary finite-index subgroups (not just
Ξ(n)
for somen
) - define the
q
-expansion as a formal power series
theorem
Function.Periodic.im_invQParam_pos_of_abs_lt_one
{h : β}
(hh : 0 < h)
{q : β}
(hq : Complex.abs q < 1)
(hq_ne : q β 0)
:
0 < (Function.Periodic.invQParam h q).im
theorem
SlashInvariantFormClass.periodic_comp_ofComplex
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[SlashInvariantFormClass F (CongruenceSubgroup.Gamma n) k]
:
Function.Periodic (βf β βUpperHalfPlane.ofComplex) βn
def
SlashInvariantFormClass.cuspFunction
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
:
The analytic function F
such that f Ο = F (exp (2 * Ο * I * Ο / n))
, extended by a choice of
limit at 0
.
Equations
- SlashInvariantFormClass.cuspFunction n f = Function.Periodic.cuspFunction (βn) (βf β βUpperHalfPlane.ofComplex)
Instances For
theorem
SlashInvariantFormClass.eq_cuspFunction
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[NeZero n]
[SlashInvariantFormClass F (CongruenceSubgroup.Gamma n) k]
(Ο : UpperHalfPlane)
:
SlashInvariantFormClass.cuspFunction n f (Function.Periodic.qParam βn βΟ) = f Ο
theorem
ModularFormClass.differentiableAt_comp_ofComplex
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
{Ξ : Subgroup (Matrix.SpecialLinearGroup (Fin 2) β€)}
(f : F)
[ModularFormClass F Ξ k]
{z : β}
(hz : 0 < z.im)
:
DifferentiableAt β (βf β βUpperHalfPlane.ofComplex) z
theorem
ModularFormClass.bounded_at_infty_comp_ofComplex
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
{Ξ : Subgroup (Matrix.SpecialLinearGroup (Fin 2) β€)}
(f : F)
[ModularFormClass F Ξ k]
:
(Filter.comap Complex.im Filter.atTop).BoundedAtFilter (βf β βUpperHalfPlane.ofComplex)
theorem
ModularFormClass.differentiableAt_cuspFunction
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[NeZero n]
[ModularFormClass F (CongruenceSubgroup.Gamma n) k]
{q : β}
(hq : Complex.abs q < 1)
:
theorem
ModularFormClass.analyticAt_cuspFunction_zero
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[NeZero n]
[ModularFormClass F (CongruenceSubgroup.Gamma n) k]
:
theorem
CuspFormClass.zero_at_infty_comp_ofComplex
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
{Ξ : Subgroup (Matrix.SpecialLinearGroup (Fin 2) β€)}
(f : F)
[CuspFormClass F Ξ k]
:
(Filter.comap Complex.im Filter.atTop).ZeroAtFilter (βf β βUpperHalfPlane.ofComplex)
theorem
CuspFormClass.cuspFunction_apply_zero
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[NeZero n]
[CuspFormClass F (CongruenceSubgroup.Gamma n) k]
:
theorem
CuspFormClass.exp_decay_atImInfty
{k : β€}
{F : Type u_1}
[FunLike F UpperHalfPlane β]
(n : β)
(f : F)
[NeZero n]
[CuspFormClass F (CongruenceSubgroup.Gamma n) k]
:
βf =O[UpperHalfPlane.atImInfty] fun (Ο : UpperHalfPlane) => Real.exp (-2 * Real.pi * Ο.im / βn)