Slash actions #
This file defines a class of slash actions, which are families of right actions of a given group
parametrized by some Type. This is modeled on the slash action of GLPos (Fin 2) ℝ
on the space
of modular forms.
Notation #
In the ModularForm
locale, this provides
f ∣[k;γ] A
: thek
thγ
-compatible slash action byA
onf
f ∣[k] A
: thek
thℂ
-compatible slash action byA
onf
; a shorthand forf ∣[k;ℂ] A
A general version of the slash action of the space of modular forms.
- map : β → G → α → α
- slash_mul (k : β) (g h : G) (a : α) : SlashAction.map γ k (g * h) a = SlashAction.map γ k h (SlashAction.map γ k g a)
- smul_slash (k : β) (g : G) (a : α) (z : γ) : SlashAction.map γ k g (z • a) = z • SlashAction.map γ k g a
- add_slash (k : β) (g : G) (a b : α) : SlashAction.map γ k g (a + b) = SlashAction.map γ k g a + SlashAction.map γ k g b
Instances
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Slash_action induced by a monoid homomorphism.
Equations
- monoidHomSlashAction h = { map := fun (k : β) (g : H) => SlashAction.map γ k (h g), zero_slash := ⋯, slash_one := ⋯, slash_mul := ⋯, smul_slash := ⋯, add_slash := ⋯ }
Instances For
The weight k
action of GL(2, ℝ)⁺
on functions f : ℍ → ℂ
.
Equations
- ModularForm.slash k γ f x = f (γ • x) * ↑(↑↑γ).det ^ (k - 1) * UpperHalfPlane.denom γ x ^ (-k)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- ModularForm.SLAction = monoidHomSlashAction (Matrix.SpecialLinearGroup.toGLPos.comp (Matrix.SpecialLinearGroup.map (Int.castRingHom ℝ)))
The constant function 1 is invariant under any element of SL(2, ℤ)
.
Variant of is_invariant_one
with the left hand side in simp normal form.
A function f : ℍ → ℂ
is slash-invariant, of weight k ∈ ℤ
and level Γ
,
if for every matrix γ ∈ Γ
we have f(γ • z)= (c*z+d)^k f(z)
where γ= ![![a, b], ![c, d]]
,
and it acts on ℍ
via Möbius transformations.