Skip to content

Commit 5a9a408

Browse files
leanprover-community-mathlib4-botmathlib4-botkim-emeric-wiesergithub-actions
authored
chore: adaptations for nightly-2025-06-05 (#25490)
* 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 * Update lean-toolchain for testing leanprover/lean4#8519 * 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 * Trigger CI for leanprover/lean4#8519 * 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 * chore: remove simp attribute when value of argument can not be inferred by simp * 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 * change phrasing of comments * chore(Geometry/Manifold): two simp-lemmas can be proven by simp * fix two lint problems * Trigger CI for leanprover/lean4#8519 * chore: bump to nightly-2025-06-03 * fix * fix * Update lean-toolchain for testing leanprover/lean4#8610 * fix * revert change in `Mathlib.Data.ZMOD.Basic` * fix Mathlib/Data/List/EditDistance/Estimator.lean * give specialized simp lemmas higher prio * simp can prove these * simp can prove these * chore: bump to nightly-2025-06-04 * bump toolchain * Adapt eqns * Revert "Adapt eqns" This reverts commit 34f1f7f. * Simply remove check for now * fix a bunch * fixes? * chore: adaptations for nightly-2025-06-04 * add `simp low` lemma `injOn_of_eq_iff_eq` * wip * wip * wip * fix * Trigger CI for leanprover-community/batteries#1220 * Merge master into nightly-testing * chore: bump to nightly-2025-06-05 * Kick CI * Bump lean4-cli * Bump import-graph * Kick CI * update lakefile * chore: use more robust syntax quotation in Shake * cleanup lakefile --------- Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Kim Morrison <[email protected]> Co-authored-by: Eric Wieser <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Joseph Rotella <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: Sebastian Ullrich <[email protected]> Co-authored-by: Johan Commelin <[email protected]> Co-authored-by: Jovan Gerbscheid <[email protected]> Co-authored-by: Joachim Breitner <[email protected]>
1 parent 004f545 commit 5a9a408

File tree

6 files changed

+13
-12
lines changed

6 files changed

+13
-12
lines changed

Mathlib/Data/BitVec.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -63,8 +63,6 @@ instance : CommSemiring (BitVec w) :=
6363
(fun _ => rfl) /- toFin_natCast -/
6464
-- The statement in the new API would be: `n#(k.succ) = ((n / 2)#k).concat (n % 2 != 0)`
6565

66-
open Fin.IntCast
67-
6866
-- TODO: move to the Lean4 repository.
6967
@[simp] theorem _root_.Fin.val_intCast {n : Nat} [NeZero n] (x : Int) :
7068
(x : Fin n).val = (x % n).toNat := by

Mathlib/Tactic/Eqns.lean

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -39,9 +39,10 @@ initialize eqnsAttribute : NameMapExtension (Array Name) ←
3939
descr := "Overrides the equation lemmas for a declaration to the provided list"
4040
add := fun
4141
| declName, `(attr| eqns $[$names]*) => do
42-
if let some _ := Meta.eqnsExt.getState (← getEnv) |>.map.find? declName then
43-
throwError "There already exist stored eqns for '{declName}'; registering new equations \
44-
will not have the desired effect."
42+
-- We used to be able to check here if equational lemmas have already been registered in
43+
-- Leans `eqsnExt`, but that has been removed in #8519, so no warning in that case.
44+
-- Now we just hope that the `GetEqnsFn` registered below will always run before
45+
-- Lean’s.
4546
names.mapM realizeGlobalConstNoOverloadWithInfo
4647
| _, _ => Lean.Elab.throwUnsupportedSyntax }
4748

Shake/Main.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -247,7 +247,9 @@ def parseHeader (srcSearchPath : SearchPath) (mod : Name) :
247247
parseHeaderFromString text path.toString
248248

249249
/-- Gets the name `Foo` in `import Foo`. -/
250-
def importId (stx : TSyntax ``Parser.Module.import) : Name := stx.raw[3].getId
250+
def importId : TSyntax ``Parser.Module.import → Name
251+
| `(Parser.Module.import| import $id) => id.getId
252+
| stx => panic! s!"unexpected syntax {stx}"
251253

252254
/-- Analyze and report issues from module `i`. Arguments:
253255

lake-manifest.json

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -24,11 +24,11 @@
2424
{"url": "https://github.com/leanprover-community/import-graph",
2525
"type": "git",
2626
"subDir": null,
27-
"scope": "leanprover-community",
28-
"rev": "e25fe66cf13e902ba550533ef681cc35a9f18dc2",
27+
"scope": "",
28+
"rev": "856a8cb8908af109aac3ce13e2b4f866f3d75199",
2929
"name": "importGraph",
3030
"manifestFile": "lake-manifest.json",
31-
"inputRev": "main",
31+
"inputRev": "nightly-testing",
3232
"inherited": false,
3333
"configFile": "lakefile.toml"},
3434
{"url": "https://github.com/leanprover-community/ProofWidgets4",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover",
78-
"rev": "a0abd472348dd725adbb26732e79b26e7e220913",
78+
"rev": "1604206fcd0462da9a241beeac0e2df471647435",
7979
"name": "Cli",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",

lakefile.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ require "leanprover-community" / "proofwidgets" @ git "v0.0.63-pre" -- ProofWidg
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."
18-
require "leanprover-community" / "importGraph" @ git "main"
18+
require "leanprover-community" / "importGraph" @ git "nightly-testing"
1919
require "leanprover-community" / "LeanSearchClient" @ git "main"
2020
require "leanprover-community" / "plausible" @ git "nightly-testing"
2121

lean-toolchain

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

0 commit comments

Comments
 (0)