Skip to content

Commit 597ea55

Browse files
committed
chore: adaptations for nightly-2025-10-20
2 parents d07fa73 + f23e0ba commit 597ea55

File tree

4 files changed

+19
-12
lines changed

4 files changed

+19
-12
lines changed

Cache/IO.lean

Lines changed: 7 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -70,7 +70,7 @@ def CURLBIN :=
7070

7171
/-- leantar version at https://github.com/digama0/leangz -/
7272
def LEANTARVERSION :=
73-
"0.1.16-pre2"
73+
"0.1.16-pre3"
7474

7575
def EXE := if System.Platform.isWindows then ".exe" else ""
7676

@@ -311,18 +311,20 @@ def mkBuildPaths (mod : Name) : CacheM <| List (FilePath × Bool) := do
311311
return [
312312
-- Note that `packCache` below requires that the `.trace` file is first in this list.
313313
(packageDir / LIBDIR / path.withExtension "trace", true),
314+
-- Note: the `.olean`, `.olean.server`, `.olean.private` files must be consecutive,
315+
-- and in this order. The corresponding `.hash` files can come afterwards, in any order.
314316
(packageDir / LIBDIR / path.withExtension "olean", true),
317+
(packageDir / LIBDIR / path.withExtension "olean.server", false),
318+
(packageDir / LIBDIR / path.withExtension "olean.private", false),
315319
(packageDir / LIBDIR / path.withExtension "olean.hash", true),
320+
(packageDir / LIBDIR / path.withExtension "olean.server.hash", false),
321+
(packageDir / LIBDIR / path.withExtension "olean.private.hash", false),
316322
(packageDir / LIBDIR / path.withExtension "ilean", true),
317323
(packageDir / LIBDIR / path.withExtension "ilean.hash", true),
318324
(packageDir / IRDIR / path.withExtension "c", true),
319325
(packageDir / IRDIR / path.withExtension "c.hash", true),
320326
-- (packageDir / LIBDIR / path.withExtension "ir", true),
321327
-- (packageDir / LIBDIR / path.withExtension "ir.hash", true),
322-
-- (packageDir / LIBDIR / path.withExtension "olean.private", false),
323-
-- (packageDir / LIBDIR / path.withExtension "olean.private.hash", false),
324-
-- (packageDir / LIBDIR / path.withExtension "olean.server", false),
325-
-- (packageDir / LIBDIR / path.withExtension "olean.server.hash", false),
326328
(packageDir / LIBDIR / path.withExtension "extra", false)]
327329

328330
/-- Check that all required build files exist. -/

Mathlib/Data/Set/Insert.lean

Lines changed: 6 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -40,7 +40,12 @@ theorem insert_def (x : α) (s : Set α) : insert x s = { y | y = x ∨ y ∈ s
4040
@[simp]
4141
theorem subset_insert (x : α) (s : Set α) : s ⊆ insert x s := fun _ => Or.inr
4242

43-
grind_pattern subset_insert => _ ⊆ insert x s
43+
-- This is a fairly aggressive pattern; it might be safer to use
44+
-- `s ⊆ insert x s` or `_ ⊆ insert x s` instead.
45+
-- Currently Cslib relies on this.
46+
-- See `MathlibTest/grind/set.lean` for a test case illustrating the reasoning
47+
-- that Cslib is relying on.
48+
grind_pattern subset_insert => insert x s
4449

4550
theorem mem_insert (x : α) (s : Set α) : x ∈ insert x s :=
4651
Or.inl rfl

lake-manifest.json

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "84b9c4f5f7f9ab594ca6252bf91e293b974cc29a",
28+
"rev": "6de2dd4b6aac9ce8825fa93c2b99b5e06c0b5456",
2929
"name": "importGraph",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "nightly-testing",
@@ -55,7 +55,7 @@
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "07d6ac02ebdf6ef77651c9e1750c179d0f609ee6",
58+
"rev": "85cc6389e0566786b2966da9512d1e8cf2402d96",
5959
"name": "Qq",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "nightly-testing",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "8d6f25c325b16b3b8a6dee0f05d20e424fe1bc30",
68+
"rev": "4ea21a7d20e5ac4db46bab6013b53edc109abd04",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "nightly-testing",
@@ -75,10 +75,10 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover",
78-
"rev": "b62fd39acc32da6fb8bb160c82d1bbc3cb3c186e",
78+
"rev": "88e435f7b94b7e77c2006a72bf0702750684a8fb",
7979
"name": "Cli",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "main",
81+
"inputRev": "nightly-testing",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"}],
8484
"name": "mathlib",

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2025-10-19
1+
leanprover/lean4:nightly-2025-10-20

0 commit comments

Comments
 (0)