Skip to content

Commit 32fc4ca

Browse files
committed
new quat alg file on the way to T
1 parent b1d0372 commit 32fc4ca

File tree

1 file changed

+90
-0
lines changed

1 file changed

+90
-0
lines changed
+90
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,90 @@
1+
/-
2+
Copyright (c) 2024 Kevin Buzzaed. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Kevin Buzzard
5+
-/
6+
import Mathlib.LinearAlgebra.Matrix.GeneralLinearGroup
7+
import Mathlib.Geometry.Manifold.Instances.UnitsOfNormedAlgebra
8+
import Mathlib
9+
10+
/-
11+
12+
# Definiteion of automorphic forms on a totally definite quaternion algebra
13+
-/
14+
15+
suppress_compilation
16+
17+
variable (F : Type*) [Field F] [NumberField F]
18+
19+
variable (D : Type*) [Ring D] [Algebra F D] [FiniteDimensional F D]
20+
21+
#check DedekindDomain.FiniteAdeleRing
22+
23+
open DedekindDomain
24+
25+
open scoped NumberField
26+
27+
#check FiniteAdeleRing (𝓞 F) F
28+
29+
-- my work (two PRs)
30+
instance : TopologicalSpace (FiniteAdeleRing (𝓞 F) F) := sorry
31+
instance : TopologicalRing (FiniteAdeleRing (𝓞 F) F) := sorry
32+
33+
open scoped TensorProduct
34+
35+
#check D ⊗[F] (FiniteAdeleRing (𝓞 F) F)
36+
37+
-- your work
38+
instance : TopologicalSpace (D ⊗[F] (FiniteAdeleRing (𝓞 F) F)) := sorry
39+
instance : TopologicalRing (D ⊗[F] (FiniteAdeleRing (𝓞 F) F)) := sorry
40+
41+
namespace TotallyDefiniteQuaternionAlgebra
42+
43+
#check Units.map
44+
45+
#synth Ring (D ⊗[F] FiniteAdeleRing (𝓞 F) F)
46+
47+
noncomputable example : D →+* (D ⊗[F] FiniteAdeleRing (𝓞 F) F) := by exact
48+
Algebra.TensorProduct.includeLeftRingHom
49+
50+
abbrev Dfx := (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ
51+
noncomputable abbrev incl : Dˣ →* Dfx F D := Units.map Algebra.TensorProduct.includeLeftRingHom.toMonoidHom
52+
53+
structure AutomorphicForm (M : Type*) [AddCommGroup M] where
54+
toFun : (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ → M
55+
left_invt : ∀ (d : Dˣ) (x : (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ),
56+
toFun (Units.map Algebra.TensorProduct.includeLeftRingHom.toMonoidHom d * x) = toFun x
57+
loc_cst : ∃ U : Subgroup (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ,
58+
IsOpen (U : Set (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ) ∧
59+
∀ (x : (D ⊗[F] (FiniteAdeleRing (𝓞 F) F))ˣ),
60+
∀ u ∈ U, toFun (x * u) = toFun x
61+
62+
namespace AutomorphicForm
63+
64+
variable (M : Type*) [AddCommGroup M]
65+
66+
instance : CoeFun (AutomorphicForm F D M) (fun _ ↦ Dfx F D → M) where
67+
coe := toFun
68+
69+
instance zero : (AutomorphicForm F D M) where
70+
toFun := 0
71+
left_invt := sorry
72+
loc_cst := sorry
73+
74+
75+
instance neg (φ : AutomorphicForm F D M) : AutomorphicForm F D M where
76+
toFun x := - φ x
77+
left_invt := sorry
78+
loc_cst := sorry
79+
80+
-- instance add
81+
82+
-- instance : AddCommGroup
83+
84+
instance : MulAction (Dfx F D) (AutomorphicForm F D M) where
85+
smul := sorry -- (g • f) (x) := f(xg) -- x(gf)=(xg)f
86+
one_smul := sorry
87+
mul_smul := sorry
88+
89+
-- if M is an R-module (e.g. if M = R!), then Automorphic forms are also an R-module
90+
-- with the action being 0on the coefficients.

0 commit comments

Comments
 (0)