Skip to content

Commit f842fc7

Browse files
committed
Bump mathlib to v4.19.0
1 parent 96f1bd1 commit f842fc7

File tree

4 files changed

+14
-14
lines changed

4 files changed

+14
-14
lines changed

LeanCamCombi/GrowthInGroups/Lecture1.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -70,7 +70,7 @@ open scoped Classical in
7070
/-- An auxiliary lemma used in the proof of the collar theorem. -/
7171
lemma proposition_1_7 :
7272
∃ ε > 0, ∀ X : Finset SL(2, ℝ), #(X ^ 2) ≤ 1000 * #X → (∀ M ∈ X, ∀ i j, |M i j| ≤ ε) →
73-
∃ A : Subgroup SL(2, ℝ), A.IsCommutative
73+
∃ A : Subgroup SL(2, ℝ), IsMulCommutative A
7474
∃ a : Fin 10000000 → SL(2, ℝ), (X : Set SL(2, ℝ)) ⊆ ⋃ i, a i • A := showcased
7575

7676
/-- The **Breuillard-Green-Tao theorem**. -/

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": "",
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.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -25,7 +25,7 @@ weak.linter.style.setOption = true
2525
linter.docPrime = false
2626
linter.hashCommand = true
2727
linter.oldObtain = true
28-
linter.refine = true
28+
weak.linter.refine = true
2929
linter.style.cdot = true
3030
linter.style.dollarSyntax = true
3131
linter.style.header = true

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.18.0
1+
leanprover/lean4:v4.19.0

0 commit comments

Comments
 (0)