Skip to content

Commit 99a77d1

Browse files
committed
Bump mathlib to v4.22.0
1 parent e8dad14 commit 99a77d1

File tree

4 files changed

+28
-28
lines changed

4 files changed

+28
-28
lines changed

LeanCamCombi/GraphTheory/ExampleSheet1.lean

Lines changed: 10 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -20,7 +20,7 @@ If you solve a question in Lean, feel free to open a Pull Request on Github!
2020

2121
open Fintype (card)
2222
open Function SimpleGraph
23-
open scoped BigOperators Cardinal
23+
open scoped Cardinal SetRel
2424

2525
namespace GraphTheory
2626
namespace ES1
@@ -208,19 +208,19 @@ all degrees of $$X$$ are finite (while degrees in $$Y$$ have no restriction)?
208208

209209
-- This translation looks slightly painful because of the `cardinal`.
210210
lemma q14_part1 :
211-
∃ r : ℕ → ℕ → Prop,
212-
(∀ A : Finset ℕ, (A.card : Cardinal) ≤ #(Rel.image r A)) ∧
213-
∀ f : ℕ → ℕ, Injective f → ∃ n, ¬ r n (f n) :=
211+
∃ r : SetRel ℕ ℕ,
212+
(∀ A : Finset ℕ, (A.card : Cardinal) ≤ #(r.image A)) ∧
213+
∀ f : ℕ → ℕ, Injective f → ∃ n, ¬ n ~[r] f n :=
214214
sorry
215215

216-
lemma q14_part2 [DecidableEq β] [Countable α] [Countable β] (r : α → β → Prop)
217-
[∀ a, Fintype (Rel.image r {a})] (hr : ∀ A : Finset α, A.card ≤ card (Rel.image r A)) :
218-
∃ f : α → β, Injective f ∧ ∀ a, r a (f a) :=
216+
lemma q14_part2 [DecidableEq β] [Countable α] [Countable β] (r : SetRel α β)
217+
[∀ a, Fintype (r.image {a})] (hr : ∀ A : Finset α, A.card ≤ card (r.image A)) :
218+
∃ f : α → β, Injective f ∧ ∀ a, a ~[r] f a :=
219219
sorry
220220

221-
lemma q14_part3 [DecidableEq β] (r : α → β → Prop) [∀ a, Fintype (Rel.image r {a})]
222-
(hr : ∀ A : Finset α, A.card ≤ card (Rel.image r A)) :
223-
∃ f : α → β, Injective f ∧ ∀ a, r a (f a) :=
221+
lemma q14_part3 [DecidableEq β] (r : SetRel α β) [∀ a, Fintype (r.image {a})]
222+
(hr : ∀ A : Finset α, A.card ≤ card (r.image A)) :
223+
∃ f : α → β, Injective f ∧ ∀ a, a ~[r] f a :=
224224
sorry
225225

226226
/-!

lake-manifest.json

Lines changed: 16 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -5,27 +5,27 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "308445d7985027f538e281e18df29ca16ede2ba3",
8+
"rev": "79e94a093aff4a60fb1b1f92d9681e407124c2ca",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.21.0",
11+
"inputRev": "v4.22.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": "c4aa78186d388e50a436e8362b947bae125a2933",
18+
"rev": "b100ad4c5d74a464f497aaa8e7c74d86bf39a56f",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": "main",
21+
"inputRev": "v4.22.0",
2222
"inherited": true,
2323
"configFile": "lakefile.toml"},
2424
{"url": "https://github.com/leanprover-community/LeanSearchClient",
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "6c62474116f525d2814f0157bb468bf3a4f9f120",
28+
"rev": "99657ad92e23804e279f77ea6dbdeebaa1317b98",
2929
"name": "LeanSearchClient",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -35,57 +35,57 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "d07bd64f1910f1cc5e4cc87b6b9c590080e7a457",
38+
"rev": "eb164a46de87078f27640ee71e6c3841defc2484",
3939
"name": "importGraph",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "main",
41+
"inputRev": "v4.22.0",
4242
"inherited": true,
4343
"configFile": "lakefile.toml"},
4444
{"url": "https://github.com/leanprover-community/ProofWidgets4",
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "6980f6ca164de593cb77cd03d8eac549cc444156",
48+
"rev": "1253a071e6939b0faf5c09d2b30b0bfc79dae407",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.62",
51+
"inputRev": "v0.0.68",
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": "8ff27701d003456fd59f13a9212431239d902aef",
58+
"rev": "1256a18522728c2eeed6109b02dd2b8f207a2a3c",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
61-
"inputRev": "master",
61+
"inputRev": "v4.22.0",
6262
"inherited": true,
6363
"configFile": "lakefile.toml"},
6464
{"url": "https://github.com/leanprover-community/quote4",
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "e9c65db4823976353cd0bb03199a172719efbeb7",
68+
"rev": "917bfa5064b812b7fbd7112d018ea0b4def25ab3",
6969
"name": "Qq",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "master",
71+
"inputRev": "v4.22.0",
7272
"inherited": true,
7373
"configFile": "lakefile.toml"},
7474
{"url": "https://github.com/leanprover-community/batteries",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "8d2067bf518731a70a255d4a61b5c103922c772e",
78+
"rev": "240676e9568c254a69be94801889d4b13f3b249f",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "main",
81+
"inputRev": "v4.22.0",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"},
8484
{"url": "https://github.com/leanprover/lean4-cli",
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "7c6aef5f75a43ebbba763b44d535175a1b04c9e0",
88+
"rev": "c682c91d2d4dd59a7187e2ab977ac25bd1f87329",
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
@@ -39,7 +39,7 @@ linter.style.setOption = true
3939
[[require]]
4040
name = "mathlib"
4141
git = "https://github.com/leanprover-community/mathlib4.git"
42-
rev = "v4.21.0"
42+
rev = "v4.22.0"
4343

4444
[[lean_lib]]
4545
name = "LeanCamCombi"

lean-toolchain

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

0 commit comments

Comments
 (0)