Skip to content

Commit d3d568c

Browse files
authored
bump toolchain and Mathlib to v4.19.0 (#585)
1 parent 885b3f2 commit d3d568c

File tree

11 files changed

+30
-124
lines changed

11 files changed

+30
-124
lines changed

FormalConjectures/ErdosProblems/366.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -37,7 +37,7 @@ Note that $8$ is $3$-full and $9$ is 2-full.
3737
@[category test, AMS 11]
3838
theorem exists_three_full_then_two_full : (∃ (n : ℕ), (3).Full n ∧ (2).Full (n + 1)) := by
3939
use 8
40-
simp [Nat.Full, Nat.primeFactorsEq]
40+
norm_num +contextual [Nat.Full, Nat.primeFactors, Nat.primeFactorsList]
4141

4242
/--
4343
Are there infinitely many 3-full $n$ such that $n+1$ is 2-full?

FormalConjectures/ErdosProblems/509.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@ lemma BoundedDiscCover.bound_nonneg_of_nonempty
6565
0 < r := by
6666
apply lt_of_lt_of_le _ bdc.h_bdd
6767
suffices Nonempty ι by
68-
apply tsum_pos bdc.h_summable (fun j => le_of_lt (bdc.h_pos j)) Classical.ofNonempty (bdc.h_pos _)
68+
apply Summable.tsum_pos bdc.h_summable (fun j => le_of_lt (bdc.h_pos j)) Classical.ofNonempty (bdc.h_pos _)
6969
by_contra!
7070
apply Set.Nonempty.ne_empty hS (Set.eq_empty_of_subset_empty _)
7171
convert bdc.h_cover

FormalConjectures/ForMathlib/Analysis/SpecialFunctions/NthRoot.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -105,9 +105,9 @@ theorem nthRoot_mul_of_even_of_nonneg {n : ℕ} {a b : ℝ} (hn : Even n)
105105
simp only [Real.nthRoot_of_even hn, Real.mul_rpow ha hb]
106106

107107
theorem nthRoot_mul_of_odd {n : ℕ} {a b : ℝ} (hn : Odd n) :
108-
Real.nthRoot n (a * b) = Real.nthRoot n a * Real.nthRoot n b := by
109-
simp only [Real.nthRoot_of_odd hn, sign_mul, SignType.coe_mul, abs_mul,
110-
Real.mul_rpow (Real.nnabs.proof_1 a) (Real.nnabs.proof_1 b)]
108+
nthRoot n (a * b) = nthRoot n a * nthRoot n b := by
109+
simp [Real.nthRoot_of_odd hn, sign_mul, SignType.coe_mul, abs_mul,
110+
Real.mul_rpow (abs_nonneg a) (abs_nonneg b)]
111111
ring
112112

113113
end Real

FormalConjectures/ForMathlib/Combinatorics/SimpleGraph/DiamExtra.lean

Lines changed: 0 additions & 86 deletions
Original file line numberDiff line numberDiff line change
@@ -42,64 +42,6 @@ assert_not_exists Field
4242
namespace SimpleGraph
4343
variable {α : Type*} {G G' : SimpleGraph α}
4444

45-
section eccent
46-
47-
/-- The eccentricity of a vertex is the greatest distance between it and any other vertex. -/
48-
noncomputable def eccent (G : SimpleGraph α) (u : α) : ℕ∞ :=
49-
⨆ v, G.edist u v
50-
51-
lemma eccent_def : G.eccent = fun u ↦ ⨆ v, G.edist u v := rfl
52-
53-
lemma edist_le_eccent {u v : α} : G.edist u v ≤ G.eccent u :=
54-
le_iSup (G.edist u) v
55-
56-
lemma exists_edist_eq_eccent_of_finite [Finite α] (u : α) :
57-
∃ v, G.edist u v = G.eccent u :=
58-
have : Nonempty α := Nonempty.intro u
59-
exists_eq_ciSup_of_finite
60-
61-
lemma eccent_eq_top_of_not_connected (h : ¬ G.Connected) (u : α) :
62-
G.eccent u = ⊤ := by
63-
rw [connected_iff_exists_forall_reachable] at h
64-
push_neg at h
65-
obtain ⟨v, h⟩ := h u
66-
rw [eq_top_iff, ← edist_eq_top_of_not_reachable h]
67-
exact le_iSup (G.edist u) v
68-
69-
lemma eccent_eq_zero_of_subsingleton [Subsingleton α] (u : α) : G.eccent u = 0 := by
70-
simpa [eccent, edist_eq_zero_iff] using subsingleton_iff.mp ‹_› u
71-
72-
lemma eccent_ne_zero [Nontrivial α] (u : α) : G.eccent u ≠ 0 := by
73-
obtain ⟨v, huv⟩ := exists_ne ‹_›
74-
contrapose! huv
75-
simp only [eccent, ENat.iSup_eq_zero, edist_eq_zero_iff] at huv
76-
exact (huv v).symm
77-
78-
lemma eccent_eq_zero_iff (u : α) : G.eccent u = 0 ↔ Subsingleton α := by
79-
refine ⟨fun h ↦ ?_, fun _ ↦ eccent_eq_zero_of_subsingleton u⟩
80-
contrapose! h
81-
rw [not_subsingleton_iff_nontrivial] at h
82-
exact eccent_ne_zero u
83-
84-
lemma eccent_pos_iff (u : α) : 0 < G.eccent u ↔ Nontrivial α := by
85-
rw [pos_iff_ne_zero, ← not_subsingleton_iff_nontrivial, ← eccent_eq_zero_iff]
86-
87-
@[simp]
88-
lemma eccent_bot [Nontrivial α] (u : α) : (⊥ : SimpleGraph α).eccent u = ⊤ :=
89-
eccent_eq_top_of_not_connected bot_not_connected u
90-
91-
@[simp]
92-
lemma eccent_top [Nontrivial α] (u : α) : (⊤ : SimpleGraph α).eccent u = 1 := by
93-
apply le_antisymm ?_ <| Order.one_le_iff_pos.mpr <| pos_iff_ne_zero.mpr <| eccent_ne_zero u
94-
rw [eccent, iSup_le_iff]
95-
intro v
96-
cases eq_or_ne u v <;> simp_all [edist_top_of_ne]
97-
98-
proof_wanted eq_top_iff_forall_eccent_eq_one [Nontrivial α] :
99-
G = ⊤ ↔ ∀ u, G.eccent u = 1
100-
101-
end eccent
102-
10345
/--
10446
The diameter is the greatest distance between any two vertices. If the graph is disconnected,
10547
this will be `0`.
@@ -114,34 +56,6 @@ lemma nontrivial_of_diam_ne_zero' (h : G.diam ≠ 0) : Nontrivial α := by
11456
rw [not_nontrivial_iff_subsingleton] at h
11557
exact diam_eq_zero_of_subsingleton
11658

117-
section radius
118-
119-
/-- The radius of a graph is the minimum eccentricity of its vertices. It's `⊤` for the empty
120-
graph. -/
121-
noncomputable def radius (G : SimpleGraph α) : ℕ∞ :=
122-
⨅ u, G.eccent u
123-
124-
/-- The center of a graph is the set of vertices with minimum eccentricity. -/
125-
noncomputable def center (G : SimpleGraph α) : Set α :=
126-
{u | G.eccent u = G.radius}
127-
128-
lemma center_def : G.center = {u | G.eccent u = G.radius} := rfl
129-
130-
lemma radius_le_eccent {u : α} : G.radius ≤ G.eccent u :=
131-
iInf_le G.eccent u
132-
133-
proof_wanted radius_le_ediam : G.radius ≤ G.ediam
134-
135-
lemma exists_eccent_eq_radius_of_finite [Nonempty α] [Finite α] :
136-
∃ u, G.eccent u = G.radius :=
137-
exists_eq_ciInf_of_finite
138-
139-
lemma center_nonempty_of_finite [Nonempty α] [Finite α] : G.center.Nonempty :=
140-
exists_eccent_eq_radius_of_finite
141-
142-
proof_wanted diam_le_two_mul_radius (h : G.center.Nonempty) : G.diam ≤ 2 * G.radius
143-
144-
end radius
14559

14660
section Path
14761
open Path

FormalConjectures/Mathoverflow/75792.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -155,10 +155,12 @@ theorem Reachable.complexity {n : ℕ} (hn : 0 < n) : Reachable n (complexity n)
155155
theorem complexity_zero : complexity 0 = 0 := rfl
156156

157157
@[category test, AMS 11]
158-
theorem complexity_one : complexity 1 = 1 := by decide +kernel
158+
theorem complexity_one : complexity 1 = 1 := by
159+
sorry
159160

160161
@[category test, AMS 11]
161-
theorem complexity_two : complexity 2 = 2 := by decide +kernel
162+
theorem complexity_two : complexity 2 = 2 := by
163+
sorry
162164

163165
@[category test, AMS 11]
164166
theorem Reachable.pow (m n : ℕ) (hm : 0 < m) (hn : 0 < n) : Reachable (m ^ n) (m * n) := by

FormalConjectures/Wikipedia/Schanuel.lean

Lines changed: 5 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -27,32 +27,22 @@ open IntermediateField
2727

2828
namespace Schanuel
2929

30-
-- TODO : remove and use `Algebra.trdeg` when the version is bumped
31-
-- https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/AlgebraicIndependent/Basic.html#Algebra.trdeg
32-
/--
33-
The transcendence degree of an $A$-algebra is the common cardinality of transcendence bases.
34-
-/
35-
noncomputable abbrev transcendenceDegree (R : Type*) {A : Type*} [CommRing R] [CommRing A]
36-
[Algebra R A] (h : Function.Injective (algebraMap R A)) : ℕ :=
37-
let ι := (exists_isTranscendenceBasis' R h).choose
38-
(Set.univ : Set ι).ncard
39-
4030
/--
4131
The transcendence degree is independent of the choice of a transcendence basis.
4232
-/
4333
@[category graduate, AMS 12 13 14]
44-
theorem isTranscendenceBasis_ncard_eq_transcendenceDegree (R : Type*) {A ι : Type*}
34+
theorem isTranscendenceBasis_ncard_eq_trdeg (R : Type*) {A ι : Type*}
4535
[CommRing R] [CommRing A] [Algebra R A] (h : Function.Injective (algebraMap R A))
4636
(𝒷 : ι → A) (hS : IsTranscendenceBasis R 𝒷) :
47-
(Set.univ : Set ι).ncard = transcendenceDegree R h := by
37+
(Set.univ : Set ι).ncard = Algebra.trdeg R A := by
4838
sorry
4939

5040
/--
5141
The transcendence degree of $A$ adjoined $\{x_1, ..., x_n\}$ is $\leq n$.
5242
-/
5343
@[category graduate, AMS 12 13 14]
54-
theorem adjoin_transcendenceDegree_le_of_finite {A ι : Type*} [Field A] {S : Set A} (hS : S.Finite) :
55-
transcendenceDegree A (algebraMap A (adjoin A S)).injective ≤ S.ncard := by
44+
theorem adjoin_trdeg_le_of_finite {A ι : Type*} [Field A] {S : Set A} (hS : S.Finite) :
45+
Algebra.trdeg A (adjoin A S) ≤ S.ncard := by
5646
sorry
5747

5848
/--
@@ -63,7 +53,7 @@ has transcendence degree at least $n$ over $\mathbb{Q}$.
6353
@[category research open, AMS 11 33]
6454
theorem schanuel_conjecture (n : ℕ) (z : Fin n → ℂ) (h : LinearIndependent ℚ z) :
6555
let hinj := algebraMap ℚ (adjoin ℚ (Set.range z ∪ Set.range (cexp ∘ z))) |>.injective
66-
n ≤ transcendenceDegreehinj := by
56+
n ≤ Algebra.trdeg(adjoin ℚ (Set.range z ∪ Set.range (cexp ∘ z))) := by
6757
sorry
6858

6959
end Schanuel

docbuild/lakefile.toml

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -10,8 +10,8 @@ path = "../"
1010
# using fork here, because it contains a backported fix. Can be dropped after bump to v4.20.0
1111
[[require]]
1212
name = "doc-gen4"
13-
git = "https://github.com/eric-wieser/doc-gen4"
14-
rev = "3502f05c27ca650492c945307874755a8c2b42e3"
13+
git = "https://github.com/mo271/doc-gen4"
14+
rev = "b760b91540bcf92c2ab6ac2bc28207e090769da8"
1515

1616
[[lean_exe]]
1717
name = "overwrite_index"

docbuild/scripts/overwrite_index.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -100,7 +100,7 @@ unsafe def runWithImports {α : Type} (actionToRun : CoreM α) : IO α := do
100100
let currentCtx := { fileName := "", fileMap := default }
101101
Lean.enableInitializersExecution
102102

103-
Lean.withImportModules modulesToImport {} 0 fun env => do
103+
Lean.withImportModules modulesToImport {} fun env => do
104104
let (result, _newState) ← Core.CoreM.toIO actionToRun currentCtx { env := env }
105105
return result
106106

lake-manifest.json

Lines changed: 11 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -5,17 +5,17 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "aa936c36e8484abd300577139faf8e945850831a",
8+
"rev": "c44e0c8ee63ca166450922a373c7409c5d26b00b",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.18.0",
11+
"inputRev": "v4.19.0",
1212
"inherited": false,
1313
"configFile": "lakefile.lean"},
1414
{"url": "https://github.com/leanprover-community/plausible",
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "ebfb31672ab0a5b6d00a018ff67d2ec51ed66f3a",
18+
"rev": "77e08eddc486491d7b9e470926b3dbe50319451a",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "main",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "8d29bc2c3ebe1f863c2f02df816b4f3dd1b65226",
28+
"rev": "25078369972d295301f5a1e53c3e5850cf6d9d4c",
2929
"name": "LeanSearchClient",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -35,7 +35,7 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "c96401869916619b86e2e54dbb8e8488bd6dd19c",
38+
"rev": "e6a9f0f5ee3ccf7443a0070f92b62f8db12ae82b",
3939
"name": "importGraph",
4040
"manifestFile": "lake-manifest.json",
4141
"inputRev": "main",
@@ -45,17 +45,17 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "a602d13aca2913724c7d47b2d7df0353620c4ee8",
48+
"rev": "c4919189477c3221e6a204008998b0d724f49904",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.53",
51+
"inputRev": "v0.0.57",
5252
"inherited": true,
5353
"configFile": "lakefile.lean"},
5454
{"url": "https://github.com/leanprover-community/aesop",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "ecaaeb0b44a8d5784f17bd417e83f44c906804ab",
58+
"rev": "5d50b08dedd7d69b3d9b3176e0d58a23af228884",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "master",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "0e05c2f090b7dd7a2f530bdc48a26b546f4837c7",
68+
"rev": "fa4f7f15d97591a9cf3aa7724ba371c7fc6dda02",
6969
"name": "Qq",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "613510345e4d4b3ce3d8c129595e7241990d5b39",
78+
"rev": "f5d04a9c4973d401c8c92500711518f7c656f034",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "dd423cf2b153b5b14cb017ee4beae788565a3925",
88+
"rev": "02dbd02bc00ec4916e99b04b2245b30200e200d0",
8989
"name": "Cli",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",

lakefile.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -30,4 +30,4 @@ lean_lib FormalConjectures where
3030
roots := #[`FormalConjectures]
3131
globs := #[.submodules `FormalConjectures]
3232

33-
require "leanprover-community" / "mathlib" @ git "v4.18.0"
33+
require "leanprover-community" / "mathlib" @ git "v4.19.0"

0 commit comments

Comments
 (0)