@@ -136,23 +136,26 @@ variable [SMulCommClass R Dˣ W]
136
136
137
137
def smul (r : R) (φ : AutomorphicForm F D R W U χ) :
138
138
AutomorphicForm F D R W U χ where
139
- toFun g := r • φ g
140
- left_invt := by simp [left_invt, smul_comm]
141
- has_character g z := by
142
- simp_all [has_character]
143
- rw [smul_comm] -- makes simp loop :-/
144
- right_invt := by simp_all [right_invt]
139
+ toFun g := r • φ g
140
+ left_invt := by simp [left_invt, smul_comm]
141
+ has_character g z := by
142
+ simp_all [has_character]
143
+ rw [smul_comm] -- makes simp loop :-/
144
+ right_invt := by simp_all [right_invt]
145
145
146
146
instance : SMul R (AutomorphicForm F D R W U χ) where
147
147
smul := smul
148
148
149
+ lemma smul_apply (r : R) (φ : AutomorphicForm F D R W U χ) (g : (D ⊗[F] FiniteAdeleRing (𝓞 F) F)ˣ) :
150
+ (r • φ) g = r • (φ g) := rfl
151
+
149
152
instance module : Module R (AutomorphicForm F D R W U χ) where
150
- one_smul := sorry
151
- mul_smul := sorry
152
- smul_zero := sorry
153
- smul_add := sorry
154
- add_smul := sorry
155
- zero_smul := sorry
153
+ one_smul g := by ext; simp [smul_apply]
154
+ mul_smul r s g := by ext; simp [smul_apply, mul_smul]
155
+ smul_zero r := by ext; simp [smul_apply]
156
+ smul_add r f g := by ext; simp [smul_apply]
157
+ add_smul r s g := by ext; simp [smul_apply, add_smul]
158
+ zero_smul g := by ext; simp [smul_apply]
156
159
157
160
158
161
end AutomorphicForm
0 commit comments