Skip to content

Commit ba3d843

Browse files
authored
Merge pull request #118 from Ruben-VandeVelde/bump
Bump mathlib
2 parents 7066ad8 + 06de52f commit ba3d843

File tree

12 files changed

+34
-35
lines changed

12 files changed

+34
-35
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 => by exact 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/GlobalLanglandsConjectures/GLnDefs.lean

+3-1
Original file line numberDiff line numberDiff line change
@@ -77,9 +77,10 @@ open scoped nonZeroDivisors
7777
noncomputable instance : Algebra R (FiniteAdeleRing R K) :=
7878
RingHom.toAlgebra ((algebraMap K (FiniteAdeleRing R K)).comp (algebraMap R K))
7979

80+
@[deprecated mul_nonZeroDivisor_mem_finiteIntegralAdeles]
8081
lemma FiniteAdeleRing.clear_denominator (a : FiniteAdeleRing R K) :
8182
∃ (b : R⁰) (c : R_hat R K), a * (b : R) = c := by
82-
sorry -- there's a nearly-done mathlib PR which proves this
83+
exact mul_nonZeroDivisor_mem_finiteIntegralAdeles a
8384

8485
#check Classical.choose (v.valuation_exists_uniformizer K)
8586

@@ -313,6 +314,7 @@ def annihilator {R} [CommSemiring R]
313314
(a : M) : Submodule R (M →ₗ[R] N) :=
314315
Submodule.compatibleMaps (Submodule.span R {a}) ⊥
315316

317+
set_option synthInstance.maxHeartbeats 40000 in
316318
/-- Automorphic forms for GL_n/Q with weight ρ. -/
317319
structure AutomorphicFormForGLnOverQ (n : ℕ) (ρ : Weight n) where
318320
toFun : GL (Fin n) (FiniteAdeleRing ℤ ℚ) × GL (Fin n) ℝ → ℂ

FLT/GlobalLanglandsConjectures/GLzero.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kevin Buzzard, Jonas Bayer
55
-/
66
import Mathlib.RingTheory.DedekindDomain.Ideal
7-
import Mathlib.RingTheory.IntegralRestrict
7+
import Mathlib.RingTheory.IntegralClosure.IntegralRestrict
88
import Mathlib.RingTheory.Ideal.QuotientOperations
99
import Mathlib.FieldTheory.Cardinality
1010
import FLT.GlobalLanglandsConjectures.GLnDefs

FLT/HIMExperiments/module_topology.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -179,13 +179,13 @@ lemma LinearMap.continuous_on_prod (f : (M × N) →ₗ[A] A) :
179179
suffices Continuous fun (⟨m, n⟩ : M × N) ↦ f (⟨m, 0⟩) + f (⟨0, n⟩) by
180180
simpa [← LinearMap.map_add, Prod.mk_add_mk, add_zero, zero_add]
181181
apply Continuous.add
182-
. refine Continuous.fst' (?_ : Continuous fun m ↦ f (m, 0))
182+
· refine Continuous.fst' (?_ : Continuous fun m ↦ f (m, 0))
183183
exact Module.continuous_linear_to_ring A
184184
({toFun := fun m ↦ f (m, 0),
185185
map_add' := by {intro x y; rw [← LinearMap.map_add, Prod.mk_add_mk, zero_add]},
186186
map_smul' := by intro m x; rw [←LinearMap.map_smul,
187187
RingHom.id_apply, Prod.smul_mk, smul_zero]})
188-
. apply @Continuous.snd' _ _ _ _ _ _ (fun n ↦ f (0, n))
188+
· apply @Continuous.snd' _ _ _ _ _ _ (fun n ↦ f (0, n))
189189
exact Module.continuous_linear_to_ring A
190190
({toFun := fun n ↦ f (0, n),
191191
map_add' := by {intro x y; rw [← LinearMap.map_add, Prod.mk_add_mk, add_zero]},

FLT/mathlibExperiments/Coalgebra/Monoid.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -210,7 +210,7 @@ lemma comp_one {A' : Type*} [CommSemiring A'] [Bialgebra R A']
210210
(f : AlgHomPoint R A' L) :
211211
f.comp (1 : AlgHomPoint R A' A') = 1 := by
212212
ext
213-
simp [one_def, Algebra.ofId_apply, Algebra.algebraMap_eq_smul_one, f.map_smul, f.map_one]
213+
simp [one_def, Algebra.ofId_apply, Algebra.algebraMap_eq_smul_one, map_smul, _root_.map_one]
214214

215215
end commutative_bialgebra
216216

FLT/mathlibExperiments/Frobenius.lean

+3-3
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jou Glasheen
55
-/
66
import Mathlib.RingTheory.DedekindDomain.Ideal
7-
import Mathlib.RingTheory.IntegralRestrict
7+
import Mathlib.RingTheory.IntegralClosure.IntegralRestrict
88
import Mathlib.RingTheory.Ideal.QuotientOperations
99
import Mathlib.FieldTheory.Cardinality
1010

@@ -49,7 +49,7 @@ In this file, I :
4949
## Notation
5050
5151
Note that, to define the `MulAction` of `L ≃ₐ[K] L` on the prime ideals of `𝓞 L : = B`,
52-
we used the restriction map `galRestrict`, defined in the file Mathlib.RingTheory.IntegralRestrict.
52+
we used the restriction map `galRestrict`, defined in the file Mathlib.RingTheory.IntegralClosure.IntegralRestrict.
5353
The definition of `galRestrict` is in terms of an 'AKLB setup'; i.e., where
5454
"`A` is an integrally closed domain; `K` is the fraction ring of `A`; `L` is
5555
a finite (separable) extension of `K`; `B` is the integral closure of
@@ -258,7 +258,7 @@ lemma crt_representative (b : B) : ∃ (y : B),
258258
apply Ideal.prime_of_isPrime (h := MapPrimestoPrimes A K L B i Q)
259259
contrapose! Q_ne_bot
260260
-- goal: (Q_ne_bot : i • Q = ⊥) → Q = ⊥
261-
apply_fun (i⁻¹ • .) at Q_ne_bot -- that's the hint it needs
261+
apply_fun (i⁻¹ • ·) at Q_ne_bot -- that's the hint it needs
262262
simpa using Q_ne_bot
263263
)
264264
(fun i _ j _ hij ↦ by

FLT/mathlibExperiments/Frobenius2.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ import Mathlib.FieldTheory.Cardinality
77
import Mathlib.RingTheory.DedekindDomain.Ideal
88
import Mathlib.RingTheory.Ideal.Pointwise
99
import Mathlib.RingTheory.Ideal.QuotientOperations
10-
import Mathlib.RingTheory.IntegralRestrict
10+
import Mathlib.RingTheory.IntegralClosure.IntegralRestrict
1111

1212
/-
1313

FLT/mathlibExperiments/HopfAlgebra/Basic.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -141,7 +141,7 @@ noncomputable instance instGroup : Group (AlgHomPoint R A L) where
141141
inv f := f.comp antipodeAlgHom
142142
mul_left_inv f := AlgHom.ext fun x ↦ by
143143
simp only [AlgHomPoint.mul_repr (repr := Coalgebra.comul_repr x), AlgHom.comp_apply,
144-
antipodeAlgHom_apply, ← f.map_mul, ← map_sum, f.commutes, Algebra.ofId_apply,
144+
antipodeAlgHom_apply, ← _root_.map_mul, ← map_sum, f.commutes, Algebra.ofId_apply,
145145
antipode_repr (repr := Coalgebra.comul_repr x), AlgHomPoint.one_def,
146146
Bialgebra.counitAlgHom_apply]
147147

FLT/mathlibExperiments/IsFrobenius.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Ivan Farabella, Amelia Livingston, Jujian Zhang, Kevin Buzzard
66
import Mathlib.Tactic
77
import Mathlib.NumberTheory.NumberField.Basic
88
import Mathlib.NumberTheory.NumberField.Discriminant
9-
import Mathlib.RingTheory.IntegralRestrict
9+
import Mathlib.RingTheory.IntegralClosure.IntegralRestrict
1010
import Mathlib.RingTheory.Ideal.QuotientOperations
1111
import Mathlib.NumberTheory.RamificationInertia
1212

lake-manifest.json

+12-12
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "937cd3219c0beffa7b623d2905707d1304da259e",
8+
"rev": "dc167d260ff7ee9849b436037add06bed15104be",
99
"name": "batteries",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "main",
@@ -15,7 +15,7 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "a7bfa63f5dddbcab2d4e0569c4cac74b2585e2c6",
18+
"rev": "71f54425e6fe0fa75f3aef33a2813a7898392222",
1919
"name": "Qq",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "master",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "622d52c803db99ff4ea4fb442c1db9e91aed944c",
28+
"rev": "0444234b4216e944d5be2ce42a25d7410c67876f",
2929
"name": "aesop",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "master",
@@ -35,27 +35,27 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "d1b33202c3a29a079f292de65ea438648123b635",
38+
"rev": "a96aee5245720f588876021b6a0aa73efee49c76",
3939
"name": "proofwidgets",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "v0.0.39",
41+
"inputRev": "v0.0.41",
4242
"inherited": true,
4343
"configFile": "lakefile.lean"},
4444
{"url": "https://github.com/leanprover/lean4-cli",
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "",
48-
"rev": "a11566029bd9ec4f68a65394e8c3ff1af74c1a29",
48+
"rev": "2cf1030dc2ae6b3632c84a09350b675ef3e347d0",
4949
"name": "Cli",
5050
"manifestFile": "lake-manifest.json",
5151
"inputRev": "main",
5252
"inherited": true,
53-
"configFile": "lakefile.lean"},
53+
"configFile": "lakefile.toml"},
5454
{"url": "https://github.com/leanprover-community/import-graph",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "68b518c9b352fbee16e6d632adcb7a6d0760e2b7",
58+
"rev": "57bd2065f1dbea5e9235646fb836c7cea9ab03b6",
5959
"name": "importGraph",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "main",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "",
68-
"rev": "90ef20a210ecd605e8036b280b6b85b9043b5447",
68+
"rev": "3dd071bc2260b3cf9a71863d0dee1242fec41522",
6969
"name": "mathlib",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": null,
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "",
88-
"rev": "9148a0a7506099963925cf239c491fcda5ed0044",
88+
"rev": "5e95f4776be5e048364f325c7e9d619bb56fb005",
8989
"name": "MD4Lean",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",
@@ -95,7 +95,7 @@
9595
"type": "git",
9696
"subDir": null,
9797
"scope": "",
98-
"rev": "f93115d0209de6db335725dee900d379f40c0317",
98+
"rev": "5c11428272fe190b7e726ebe448f93437d057b74",
9999
"name": "UnicodeBasic",
100100
"manifestFile": "lake-manifest.json",
101101
"inputRev": "main",
@@ -115,7 +115,7 @@
115115
"type": "git",
116116
"subDir": null,
117117
"scope": "",
118-
"rev": "b941c425f6f0f1dc45fe13b850ffa7db1bb20d04",
118+
"rev": "6d8e3118ab526f8dfcabcbdf9f05dc34e5c423a8",
119119
"name": "«doc-gen4»",
120120
"manifestFile": "lake-manifest.json",
121121
"inputRev": "main",

lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.10.0-rc2
1+
leanprover/lean4:v4.11.0-rc1

0 commit comments

Comments
 (0)