Skip to content

Commit fb92dbf

Browse files
committed
Merge branch 'main' of github.com:ImperialCollegeLondon/FLT
2 parents a0d6a47 + 828a882 commit fb92dbf

File tree

2 files changed

+11
-6
lines changed

2 files changed

+11
-6
lines changed

FLT/AutomorphicForm/QuaternionAlgebra.lean

+9-6
Original file line numberDiff line numberDiff line change
@@ -144,13 +144,16 @@ def smul (r : R) (φ : AutomorphicForm F D R W U χ) :
144144
instance : SMul R (AutomorphicForm F D R W U χ) where
145145
smul := smul
146146

147+
lemma smul_apply (r : R) (φ : AutomorphicForm F D R W U χ) (g : (D ⊗[F] FiniteAdeleRing (𝓞 F) F)ˣ) :
148+
(r • φ) g = r • (φ g) := rfl
149+
147150
instance module : Module R (AutomorphicForm F D R W U χ) where
148-
one_smul := sorry
149-
mul_smul := sorry
150-
smul_zero := sorry
151-
smul_add := sorry
152-
add_smul := sorry
153-
zero_smul := sorry
151+
one_smul g := by ext; simp [smul_apply]
152+
mul_smul r s g := by ext; simp [smul_apply, mul_smul]
153+
smul_zero r := by ext; simp [smul_apply]
154+
smul_add r f g := by ext; simp [smul_apply]
155+
add_smul r s g := by ext; simp [smul_apply, add_smul]
156+
zero_smul g := by ext; simp [smul_apply]
154157

155158

156159
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)