Skip to content

Commit bd65b29

Browse files
Module structure on TotallyDefiniteQuaternionAlgebra.AutomorphicForm
1 parent aa6dd4c commit bd65b29

File tree

2 files changed

+17
-12
lines changed

2 files changed

+17
-12
lines changed

FLT/AutomorphicForm/QuaternionAlgebra.lean

+15-12
Original file line numberDiff line numberDiff line change
@@ -136,23 +136,26 @@ variable [SMulCommClass R Dˣ W]
136136

137137
def smul (r : R) (φ : AutomorphicForm F D R W U χ) :
138138
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]
145145

146146
instance : SMul R (AutomorphicForm F D R W U χ) where
147147
smul := smul
148148

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+
149152
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]
156159

157160

158161
end AutomorphicForm

blueprint/src/chapter/QuaternionAlgebraProject.tex

+2
Original file line numberDiff line numberDiff line change
@@ -98,6 +98,7 @@ \section{Introduction and goal}
9898
\lean{TotallyDefiniteQuaternionAlgebra.AutomorphicForm.addCommGroup}
9999
\label{TotallyDefiniteQuaternionAlgebra.AutomorphicForm.addCommGroup}
100100
\uses{TotallyDefiniteQuaternionAlgebra.AutomorphicForm}
101+
\leanok
101102
Pointwise addition $(f_1+f_2)(g):=f_1(g)+f_2(g)$ makes $S_{W,\chi}(U;R)$ into an additive
102103
abelian group.
103104
\end{definition}
@@ -107,6 +108,7 @@ \section{Introduction and goal}
107108
\label{TotallyDefiniteQuaternionAlgebra.AutomorphicForm.module}
108109
\uses{TotallyDefiniteQuaternionAlgebra.AutomorphicForm,
109110
TotallyDefiniteQuaternionAlgebra.AutomorphicForm.addCommGroup}
111+
\leanok
110112
Pointwise scalar multiplication $(r\cdot f)(g):= r\cdot(f(g))$ makes
111113
$S_{W,\chi}(U;R)$ into an $R$-module.
112114
\end{definition}

0 commit comments

Comments
 (0)