Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
notation
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed May 3, 2023
1 parent 41255a4 commit d1c29ed
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/number_theory/modular_forms/slash_invariant_forms.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,7 +85,7 @@ instance slash_invariant_form_class.coe_to_fun [slash_invariant_form_class F Γ
has_coe_to_fun F (λ _, ℍ → ℂ) := fun_like.has_coe_to_fun

@[simp] lemma slash_action_eqn [slash_invariant_form_class F Γ k] (f : F) (γ : Γ) :
slash_action.map k γ ⇑f = ⇑f := slash_invariant_form_class.slash_action_eq f γ
⇑f ∣[k] γ = ⇑f := slash_invariant_form_class.slash_action_eq f γ

lemma slash_action_eqn' (k : ℤ) (Γ : subgroup SL(2, ℤ)) [slash_invariant_form_class F Γ k] (f : F)
(γ : Γ) (z : ℍ) : f (γ • z) = ((↑ₘ[ℤ]γ 1 0 : ℂ) * z +(↑ₘ[ℤ]γ 1 1 : ℂ))^k * f z :=
Expand Down

0 comments on commit d1c29ed

Please sign in to comment.