Skip to content

Commit

Permalink
bump toolchain; remove deleted imports
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 14, 2024
1 parent 5ee6767 commit 0fc755a
Show file tree
Hide file tree
Showing 5 changed files with 5 additions and 7 deletions.
1 change: 0 additions & 1 deletion ImportGraph/Gexf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Jon Eugster
-/

import Lean
import Batteries.Lean.NameMap
import Batteries.Tactic.OpenPrivate

open Lean
Expand Down
1 change: 0 additions & 1 deletion ImportGraph/Imports.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison
-/
import Lean
import Batteries.Lean.NameMap
import ImportGraph.RequiredModules

/-!
Expand Down
6 changes: 3 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover",
"rev": "726b3c9ad13acca724d4651f14afc4804a7b0e4d",
"rev": "0c8ea32a15a4f74143e4e1e107ba2c412adb90fd",
"name": "Cli",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -15,10 +15,10 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "76e9ebe4176d29cb9cc89c669ab9f1ce32b33c3d",
"rev": "2ed85f320805f9d3a455ced3b181562ed146bc20",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inputRev": "nightly-testing",
"inherited": false,
"configFile": "lakefile.toml"}],
"name": "importGraph",
Expand Down
2 changes: 1 addition & 1 deletion lakefile.toml
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ rev = "main"
[[require]]
name = "batteries"
scope = "leanprover-community"
rev = "main"
rev = "nightly-testing"

[[lean_lib]]
name = "ImportGraph"
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.14.0-rc1
leanprover/lean4:nightly-2024-11-14

0 comments on commit 0fc755a

Please sign in to comment.