Skip to content

Commit

Permalink
Prove some easy sorries in QuaternionAlgebra.NumberField (#358)
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde authored Feb 27, 2025
1 parent 957f461 commit 7cdebc8
Showing 1 changed file with 8 additions and 8 deletions.
16 changes: 8 additions & 8 deletions FLT/QuaternionAlgebra/NumberField.lean
Original file line number Diff line number Diff line change
Expand Up @@ -59,11 +59,11 @@ def DedekindDomain.ProdAdicCompletions.toAdicCompletion
(v : HeightOneSpectrum (𝓞 F)) :
ProdAdicCompletions (𝓞 F) F →ₐ[F] v.adicCompletion F where
toFun k := k v
map_one' := sorry
map_mul' := sorry
map_zero' := sorry
map_add' := sorry
commutes' := sorry
map_one' := rfl
map_mul' _ _ := rfl
map_zero' := rfl
map_add' _ _ := rfl
commutes' _ := rfl

namespace DedekindDomain.FiniteAdeleRing

Expand All @@ -88,9 +88,9 @@ def GL2.TameLevel (S : Finset (HeightOneSpectrum (𝓞 F))) :
Subgroup (GL (Fin 2) (FiniteAdeleRing (𝓞 F) F)) where
carrier := {x | (∀ v, GL2.toAdicCompletion v x ∈ GL2.localFullLevel v) ∧
(∀ v ∈ S, GL2.toAdicCompletion v x ∈ GL2.localTameLevel v)}
mul_mem' := sorry
one_mem' := sorry
inv_mem' := sorry
mul_mem' {a b} ha hb := by simp_all [mul_mem]
one_mem' := by simp_all [one_mem]
inv_mem' {x} hx := by simp_all

noncomputable def QuaternionAlgebra.TameLevel (r : Rigidification F D)
(S : Finset (HeightOneSpectrum (𝓞 F))) :
Expand Down

0 comments on commit 7cdebc8

Please sign in to comment.