Skip to content

Commit a94cef6

Browse files
bump
1 parent e75f135 commit a94cef6

File tree

5 files changed

+17
-15
lines changed

5 files changed

+17
-15
lines changed

FltRegular/FltThree/Edwards.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -513,7 +513,7 @@ theorem step5'
513513
by
514514
rw [Nat.even_mul] at this
515515
apply this.resolve_left
516-
norm_num; decide
516+
decide
517517
rw [← evenFactorExp.pow r 3, hcube]
518518
exact factors_2_even' hcoprime
519519
calc

FltRegular/NumberTheory/Cyclotomic/CyclRat.lean

-4
Original file line numberDiff line numberDiff line change
@@ -358,7 +358,6 @@ theorem dvd_last_coeff_cycl_integer [hp : Fact (p : ℕ).Prime] {ζ : 𝓞 L}
358358
← (Fin.castOrderIso hdim).toEquiv.sum_comp] at hy
359359
simp only [RelIso.coe_fn_toEquiv, Fin.coe_cast, mul_neg, ← Subtype.coe_inj, Fin.coe_castSucc,
360360
Fin.coe_orderIso_apply] at hy
361-
push_cast at hy
362361
conv_lhs at hy =>
363362
congr; rfl; ext x
364363
rw [smul_neg]
@@ -369,7 +368,6 @@ theorem dvd_last_coeff_cycl_integer [hp : Fact (p : ℕ).Prime] {ζ : 𝓞 L}
369368
conv_lhs at hy =>
370369
congr; rfl; ext x
371370
rw [← show ∀ y, _ = _ from fun y => congr_fun b.coe_basis y, ← sub_eq_add_neg]
372-
norm_cast at hy
373371
rw [sum_sub_distrib] at hy
374372
replace hy := congr_arg (b.basis.coord ((Fin.castOrderIso hdim.symm) ⟨i, hi⟩)) hy
375373
rw [← b.basis.equivFun_symm_apply, ← b.basis.equivFun_symm_apply, LinearMap.map_sub,
@@ -410,7 +408,6 @@ theorem dvd_coeff_cycl_integer (hp : (p : ℕ).Prime) {ζ : 𝓞 L} (hζ : IsPri
410408
← (Fin.castOrderIso hdim).toEquiv.sum_comp] at hy
411409
simp only [RelIso.coe_fn_toEquiv, Fin.coe_cast, mul_neg, ← Subtype.coe_inj, Fin.coe_castSucc,
412410
Fin.coe_orderIso_apply] at hy
413-
push_cast at hy
414411
conv_lhs at hy =>
415412
congr; rfl; ext x
416413
rw [smul_neg]
@@ -421,7 +418,6 @@ theorem dvd_coeff_cycl_integer (hp : (p : ℕ).Prime) {ζ : 𝓞 L} (hζ : IsPri
421418
conv_lhs at hy =>
422419
congr; rfl; ext x
423420
rw [← show ∀ y, _ = _ from fun y => congr_fun b.coe_basis y, ← sub_eq_add_neg]
424-
norm_cast at hy
425421
rw [sum_sub_distrib] at hy
426422
replace hy := congr_arg (b.basis.coord ((Fin.castOrderIso hdim.symm) ⟨j, hj⟩)) hy
427423
rw [← b.basis.equivFun_symm_apply, ← b.basis.equivFun_symm_apply, LinearMap.map_sub,

FltRegular/NumberTheory/Cyclotomic/GaloisActionOnCyclo.lean

-1
Original file line numberDiff line numberDiff line change
@@ -71,7 +71,6 @@ theorem embedding_conj (x : K) (φ : K →+* ℂ) : conj (φ x) = φ (galConj K
7171
suffices φ (galConj K p ζ) = conj (φ ζ)
7272
by
7373
rw [← Function.funext_iff]
74-
congr
7574
rw [DFunLike.coe_fn_eq]
7675
apply (hζ.powerBasis ℚ).rat_hom_ext
7776
exact this.symm

lake-manifest.json

+15-8
Original file line numberDiff line numberDiff line change
@@ -1,10 +1,11 @@
1-
{"version": "1.0.0",
1+
{"version": "1.1.0",
22
"packagesDir": ".lake/packages",
33
"packages":
44
[{"url": "https://github.com/leanprover-community/batteries",
55
"type": "git",
66
"subDir": null,
7-
"rev": "47e4cc5c5800c07d9bf232173c9941fa5bf68589",
7+
"scope": "leanprover-community",
8+
"rev": "bba0af6e930ebcbabfacf021b21dd881d58aaa9d",
89
"name": "batteries",
910
"manifestFile": "lake-manifest.json",
1011
"inputRev": "main",
@@ -13,6 +14,7 @@
1314
{"url": "https://github.com/leanprover-community/quote4",
1415
"type": "git",
1516
"subDir": null,
17+
"scope": "leanprover-community",
1618
"rev": "a7bfa63f5dddbcab2d4e0569c4cac74b2585e2c6",
1719
"name": "Qq",
1820
"manifestFile": "lake-manifest.json",
@@ -22,7 +24,8 @@
2224
{"url": "https://github.com/leanprover-community/aesop",
2325
"type": "git",
2426
"subDir": null,
25-
"rev": "882561b77bd2aaa98bd8665a56821062bdb3034c",
27+
"scope": "leanprover-community",
28+
"rev": "a64fe24aa94e21404940e9217363a9a1ed9a33a6",
2629
"name": "aesop",
2730
"manifestFile": "lake-manifest.json",
2831
"inputRev": "master",
@@ -31,25 +34,28 @@
3134
{"url": "https://github.com/leanprover-community/ProofWidgets4",
3235
"type": "git",
3336
"subDir": null,
34-
"rev": "fc8f85bab627d5196b2342bd2f08c0ace749ec89",
37+
"scope": "leanprover-community",
38+
"rev": "d1b33202c3a29a079f292de65ea438648123b635",
3539
"name": "proofwidgets",
3640
"manifestFile": "lake-manifest.json",
37-
"inputRev": "v0.0.37",
41+
"inputRev": "v0.0.39",
3842
"inherited": true,
3943
"configFile": "lakefile.lean"},
4044
{"url": "https://github.com/leanprover/lean4-cli",
4145
"type": "git",
4246
"subDir": null,
47+
"scope": "",
4348
"rev": "a11566029bd9ec4f68a65394e8c3ff1af74c1a29",
4449
"name": "Cli",
4550
"manifestFile": "lake-manifest.json",
4651
"inputRev": "main",
4752
"inherited": true,
4853
"configFile": "lakefile.lean"},
49-
{"url": "https://github.com/leanprover-community/import-graph.git",
54+
{"url": "https://github.com/leanprover-community/import-graph",
5055
"type": "git",
5156
"subDir": null,
52-
"rev": "1588be870b9c76fe62286e8f42f0b4dafa154c96",
57+
"scope": "leanprover-community",
58+
"rev": "d366a602cc4a325a6f9db3a3991dfa6d6cf409c5",
5359
"name": "importGraph",
5460
"manifestFile": "lake-manifest.json",
5561
"inputRev": "main",
@@ -58,7 +64,8 @@
5864
{"url": "https://github.com/leanprover-community/mathlib4.git",
5965
"type": "git",
6066
"subDir": null,
61-
"rev": "397d87803ee60c11623fdd680199366acaaedaef",
67+
"scope": "",
68+
"rev": "898cc8d139a9a03ab46f727f0ba5a68588774148",
6269
"name": "mathlib",
6370
"manifestFile": "lake-manifest.json",
6471
"inputRev": null,

lean-toolchain

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

0 commit comments

Comments
 (0)