Skip to content

Commit 720ebfd

Browse files
committed
Merge remote-tracking branch 'upstream/main' into golf-proofs
2 parents a39f7bd + 10e7f80 commit 720ebfd

18 files changed

+554
-46
lines changed

FLT/AutomorphicForm/QuaternionAlgebra.lean

+4-4
Original file line numberDiff line numberDiff line change
@@ -40,11 +40,11 @@ instance : Algebra A (D ⊗[R] A) :=
4040
simp only [AlgHom.toRingHom_eq_coe, RingHom.coe_coe, Algebra.TensorProduct.includeRight_apply]
4141
intro a b
4242
apply TensorProduct.induction_on (motive := fun b ↦ 1 ⊗ₜ[R] a * b = b * 1 ⊗ₜ[R] a)
43-
. simp only [mul_zero, zero_mul]
44-
. intro d a'
43+
· simp only [mul_zero, zero_mul]
44+
· intro d a'
4545
simp only [Algebra.TensorProduct.tmul_mul_tmul, one_mul, mul_one]
4646
rw [NonUnitalCommSemiring.mul_comm]
47-
. intro x y hx hy
47+
· intro x y hx hy
4848
rw [left_distrib, hx, hy, right_distrib]
4949
)
5050

@@ -205,6 +205,6 @@ lemma sMul_eval (g : Dfx F D) (f : AutomorphicForm F D M) (x : (D ⊗[F] FiniteA
205205
(g • f) x = f (x * g) := rfl
206206

207207
instance : MulAction (Dfx F D) (AutomorphicForm F D M) where
208-
smul := (..)
208+
smul := (··)
209209
one_smul := by intros; ext; simp only [sMul_eval, mul_one]
210210
mul_smul := by intros; ext; simp only [sMul_eval, mul_assoc]

FLT/AutomorphicRepresentation/Example.lean

+4-7
Original file line numberDiff line numberDiff line change
@@ -54,9 +54,6 @@ lemma ext (x y : ZHat) (h : ∀ n : ℕ+, x n = y n) : x = y := by
5454
ext n
5555
apply h
5656

57-
lemma ext_iff (x y : ZHat) : (∀ n : ℕ+, x n = y n) ↔ x = y :=
58-
⟨ext x y, fun h n => congrFun (congrArg DFunLike.coe h) n⟩
59-
6057
@[simp] lemma zero_val (n : ℕ+) : (0 : ZHat) n = 0 := rfl
6158
@[simp] lemma one_val (n : ℕ+) : (1 : ZHat) n = 1 := rfl
6259
@[simp] lemma ofNat_val (m : ℕ) [m.AtLeastTwo] (n : ℕ+) :
@@ -75,7 +72,7 @@ lemma zeroNeOne : (0 : ZHat) ≠ 1 := by
7572
instance nontrivial : Nontrivial ZHat := ⟨0, 1, zeroNeOne⟩
7673

7774
instance charZero : CharZero ZHat := ⟨ fun a b h ↦ by
78-
rw [ext_iff] at h
75+
rw [ZHat.ext_iff] at h
7976
specialize h ⟨_, (max a b).succ_pos⟩
8077
apply_fun ZMod.val at h
8178
rwa [natCast_val, ZMod.val_cast_of_lt, natCast_val, ZMod.val_cast_of_lt] at h
@@ -200,8 +197,7 @@ lemma torsionfree (N : ℕ+) : Function.Injective (fun z : ZHat ↦ N * z) := by
200197
rw [← AddMonoidHom.coe_mulLeft, injective_iff_map_eq_zero]
201198
intro a ha
202199
rw [AddMonoidHom.coe_mulLeft] at ha
203-
rw [← ext_iff]
204-
intro j
200+
ext j
205201
rw [zero_val, ← a.prop j (N * j) (by simp)]
206202
apply torsionfree_aux
207203
apply Nat.dvd_of_mul_dvd_mul_left N.pos
@@ -824,7 +820,8 @@ lemma exists_near (a : ℍ) : ∃ q : 𝓞, dist a (toQuaternion q) < 1 := by
824820
rw [add_eq_zero_iff' (by positivity) (by positivity)]
825821
rw [add_eq_zero_iff' (by positivity) (by positivity)]
826822
rw [add_eq_zero_iff' (by positivity) (by positivity)]
827-
simp_rw [and_assoc, sq_eq_zero_iff, sub_re, sub_imI, sub_imJ, sub_imK, sub_eq_zero, ← ext_iff]
823+
simp_rw [and_assoc, sq_eq_zero_iff, sub_re, sub_imI, sub_imJ, sub_imK, sub_eq_zero,
824+
← Quaternion.ext_iff]
828825
symm
829826
apply leftInvOn_toQuaternion_fromQuaternion
830827
· simp only [Set.mem_setOf]

FLT/FLT_files.lean

+1-5
Original file line numberDiff line numberDiff line change
@@ -1,13 +1,9 @@
11
import FLT.Basic.Reductions
22
import FLT.EllipticCurve.Torsion
3-
import FLT.for_mathlib.Coalgebra.Monoid
4-
import FLT.for_mathlib.Coalgebra.Sweedler
5-
import FLT.for_mathlib.Coalgebra.TensorProduct
6-
import FLT.for_mathlib.HopfAlgebra.Basic
7-
import FLT.for_mathlib.IsCentralSimple
83
import FLT.GaloisRepresentation.HardlyRamified
94
import FLT.GlobalLanglandsConjectures.GLnDefs
105
import FLT.GroupScheme.FiniteFlat
116
import FLT.Hard.Results
127
import FLT.TateCurve.TateCurve
138
import FLT.AutomorphicRepresentation.Example
9+
import FLT.mathlibExperiments.IsCentralSimple

0 commit comments

Comments
 (0)