Skip to content

Commit 3780f5f

Browse files
leanprover-community-mathlib4-botkim-emgithub-actionsmathlib4-botVierkantor
authored
chore: adaptations for nightly-2025-06-04 (#25431)
* Update lean-toolchain for testing leanprover/lean4#8347 * fixes for leanprover/lean4#8347 * Update lean-toolchain for testing leanprover/lean4#8397 * deprecations for leanprover/lean4#8397 * chore: bump to nightly-2025-05-19 * chore: adaptations for nightly-2025-05-19 * Trigger CI for leanprover/lean4#8347 * Update the style linter to use LinterOptions * Fix test * chore: adaptations for nightly-2025-05-19 (#25017) Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: Sebastian Ullrich <[email protected]> * chore: bump to nightly-2025-05-20 * Merge master into nightly-testing * feat: a `grind` test case (#25037) Adds a test case for `grind` that was previously failing in the presence of Mathlib's typeclass shortcuts. Let's just keep it in Mathlib as a regression test. Note that this is a PR to `bump/v4.21.0`, as it requires a recent nightly toolchain. (It can still be reviewed and bors'd as any other PR.) * lake update * fixes * fixes * fixes * fixes * fix * fixes * fixes * shake --update * chore: bump to nightly-2025-05-21 * Update lean-toolchain for testing leanprover/lean4#7352 * lake update * Trigger CI for leanprover/lean4#7352 * chore: adaptations for nightly-2025-05-21 * chore: adaptations for nightly-2025-05-21 (#25079) Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> * chore: adaptations for nightly-2025-05-21 * fix for leanprover/lean4#7352 * remove unneeded List.ofFn_succ from simp sets * Merge master into nightly-testing * Merge master into nightly-testing * Revert "fix for leanprover/lean4#7352" This reverts commit 38ca408. * chore: fix some defeq abuse in theorem statements around the `Id` monad (#25098) Follows on from leanprover/lean4#7352. This also deprecates: * `id.mk`, which looks like a porting error * `Free(Add)(Magma|Semigroup).mul_map_seq`, which is a garbage lemma that both is not meaningfully about the free objects and has defeq abuse everywhere. * chore: bump to nightly-2025-05-22 * update batteries * chore: bump to nightly-2025-05-23 * Update lean-toolchain for testing leanprover/lean4#8449 * chore: adaptations for nightly-2025-05-22 (#25110) Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: github-actions <[email protected]> * remove now upstreamed `clear_value` * Update lean-toolchain for testing leanprover/lean4#8457 * chore: update tests for `Format` bug fix * Trigger CI for leanprover/lean4#8457 * lake update * lake update * fixes * Merge master into nightly-testing * chore: bump to nightly-2025-05-24 * fix * chore: adaptations for nightly-2025-05-24 (#25147) Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: Eric Wieser <[email protected]> Co-authored-by: github-actions <[email protected]> * chore: adaptations for nightly-2025-05-24 * Merge master into nightly-testing * Update lean-toolchain for testing leanprover/lean4#8470 * chore: bump to nightly-2025-05-25 * chore: adaptations for nightly-2025-05-25 * chore: adaptations for nightly-2025-05-25 (#25184) Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Eric Wieser <[email protected]> Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: github-actions <[email protected]> * unsimp `List.getElem?_length` This is solved using `getElem?_neg` now. * chore: adaptations for nightly-2025-05-25 * Trigger CI for leanprover/lean4#8470 * chore: bump to nightly-2025-05-26 * lake update * deprecations * Trigger CI for leanprover/lean4#8449 * Merge master into nightly-testing * chore: bump to nightly-2025-05-27 * chore: adaptations for nightly-2025-05-27 * Update lean-toolchain for testing leanprover/lean4#8504 * chore: bump to nightly-2025-05-28 * chore: adaptations for nightly-2025-05-27 (#25234) Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Kim Morrison <[email protected]> * fix * fix merge * fix merge again * deprecations * deprecations * fix Archive * comment out test * Fix and re-enable directory dependency lint test. * chore: bump to nightly-2025-05-29 * Use the formatting from the master branch. (Seems to have been a merge that went wrong.) * lake update * chore: adaptations for nightly-2025-05-28 (#25295) Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> * fix * Trigger CI for leanprover/lean4#8337 * fixes * Merge master into nightly-testing * chore: bump to nightly-2025-05-30 * chore: adaptations for nightly-2025-05-29 (#25306) Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Rob23oba <[email protected]> * chore: bump to nightly-2025-05-31 * chore: bump to nightly-2025-06-01 * fix Archive * chore: adaptations for nightly-2025-06-01 (#25355) Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> * chore: bump to nightly-2025-06-02 * chore: adaptations for nightly-2025-06-02 (#25360) Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: github-actions <[email protected]> * Update lean-toolchain for testing leanprover/lean4#8584 * chore: adaptations for nightly-2025-06-02 * chore: bump to nightly-2025-06-03 * fix * fix * Update lean-toolchain for testing leanprover/lean4#8610 * fix * chore: bump to nightly-2025-06-04 * bump toolchain --------- Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: Sebastian Ullrich <[email protected]> Co-authored-by: Eric Wieser <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Joseph Rotella <[email protected]>
1 parent 9fbd068 commit 3780f5f

File tree

5 files changed

+19
-21
lines changed

5 files changed

+19
-21
lines changed

Mathlib/Data/Int/Order/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -16,8 +16,6 @@ open Nat
1616

1717
namespace Int
1818

19-
export private decNonneg from Init.Data.Int.Basic
20-
2119
theorem le.elim {a b : ℤ} (h : a ≤ b) {P : Prop} (h' : ∀ n : ℕ, a + ↑n = b → P) : P :=
2220
Exists.elim (le.dest h) h'
2321

Mathlib/Lean/Name.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -58,10 +58,10 @@ def Lean.Name.decapitalize (n : Name) : Name :=
5858
/-- Whether the lemma has a name of the form produced by `Lean.Meta.mkAuxLemma`. -/
5959
def Lean.Name.isAuxLemma (n : Name) : Bool :=
6060
match n with
61-
| .str _ s => "_proof_".isPrefixOf s
61+
-- `mkAuxLemma` generally allows for arbitrary prefixes but these are the ones produced by core.
62+
| .str _ s => "_proof_".isPrefixOf s || "_simp_".isPrefixOf s
6263
| _ => false
6364

64-
/-- Unfold all lemmas created by `Lean.Meta.mkAuxLemma`.
65-
The names of these lemmas end in `_auxLemma.nn` where `nn` is a number. -/
65+
/-- Unfold all lemmas created by `Lean.Meta.mkAuxLemma`. -/
6666
def Lean.Meta.unfoldAuxLemmas (e : Expr) : MetaM Expr := do
6767
deltaExpand e Lean.Name.isAuxLemma

lake-manifest.json

Lines changed: 11 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -5,10 +5,10 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "91ce5a8051438870cbb4e3c68cd12e23ace713b1",
8+
"rev": "fde3fc21dd68a10791dea22b6f5b53c5a5a5962d",
99
"name": "plausible",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "main",
11+
"inputRev": "nightly-testing",
1212
"inherited": false,
1313
"configFile": "lakefile.toml"},
1414
{"url": "https://github.com/leanprover-community/LeanSearchClient",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "d554d45b37832f5f8e8797ac0b00be585c8aea49",
28+
"rev": "e25fe66cf13e902ba550533ef681cc35a9f18dc2",
2929
"name": "importGraph",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -35,27 +35,27 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "7518acaafc0ba29be6de6c3f37637fe4148b72cb",
38+
"rev": "2d6d124aedc3023506a67e50bfd5582384d6bd17",
3939
"name": "proofwidgets",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "v0.0.61",
41+
"inputRev": "v0.0.63-pre",
4242
"inherited": false,
4343
"configFile": "lakefile.lean"},
4444
{"url": "https://github.com/leanprover-community/aesop",
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "c548baa6d2ed727c6e9b30ff627b7c67fda4a54c",
48+
"rev": "c37af3a23d5798c560bce190bfd779710eaff1e1",
4949
"name": "aesop",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "master",
51+
"inputRev": "nightly-testing",
5252
"inherited": false,
5353
"configFile": "lakefile.toml"},
5454
{"url": "https://github.com/leanprover-community/quote4",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "f827c08bdd5044b75f0fdc3178c0c600e818b76f",
58+
"rev": "e1d2994e0acdee2f0c03c9d84d28a5df34aa0020",
5959
"name": "Qq",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "master",
@@ -65,17 +65,17 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "3aafa48516440d6038efb626660c74dec6e640da",
68+
"rev": "3253675d6329e9c1ad6f762e8989f4b8a28ffa8f",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "main",
71+
"inputRev": "nightly-testing",
7272
"inherited": false,
7373
"configFile": "lakefile.toml"},
7474
{"url": "https://github.com/leanprover/lean4-cli",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover",
78-
"rev": "1606fed39cd8bd366f8a192e6558972af869efa6",
78+
"rev": "a0abd472348dd725adbb26732e79b26e7e220913",
7979
"name": "Cli",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",

lakefile.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -7,17 +7,17 @@ open Lake DSL
77
## Mathlib dependencies on upstream projects
88
-/
99

10-
require "leanprover-community" / "batteries" @ git "main"
10+
require "leanprover-community" / "batteries" @ git "nightly-testing"
1111
require "leanprover-community" / "Qq" @ git "master"
12-
require "leanprover-community" / "aesop" @ git "master"
13-
require "leanprover-community" / "proofwidgets" @ git "v0.0.62" -- ProofWidgets should always be pinned to a specific version
12+
require "leanprover-community" / "aesop" @ git "nightly-testing"
13+
require "leanprover-community" / "proofwidgets" @ git "v0.0.63-pre" -- ProofWidgets should always be pinned to a specific version
1414
with NameMap.empty.insert `errorOnBuild
1515
"ProofWidgets not up-to-date. \
1616
Please run `lake exe cache get` to fetch the latest ProofWidgets. \
1717
If this does not work, report your issue on the Lean Zulip."
1818
require "leanprover-community" / "importGraph" @ git "main"
1919
require "leanprover-community" / "LeanSearchClient" @ git "main"
20-
require "leanprover-community" / "plausible" @ git "main"
20+
require "leanprover-community" / "plausible" @ git "nightly-testing"
2121

2222
/-!
2323
## Options for building mathlib

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2025-06-02
1+
leanprover/lean4:nightly-2025-06-04

0 commit comments

Comments
 (0)