Skip to content

Commit

Permalink
Merge pull request #56 from leanprover-community/batteries
Browse files Browse the repository at this point in the history
chore: update Std->Batteries
  • Loading branch information
semorrison committed May 7, 2024
2 parents fe1eff5 + f102909 commit e6b6247
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion ProofWidgets/Demos/SelectInsertConv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Robin Böhne, Wojciech Nawrocki, Patrick Massot
-/
import Lean.Meta.ExprLens
import Std.Lean.Position
import Batteries.Lean.Position
import ProofWidgets.Data.Html
import ProofWidgets.Component.OfRpcMethod
import ProofWidgets.Component.MakeEditLink
Expand Down
6 changes: 3 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
@@ -1,11 +1,11 @@
{"version": 7,
"packagesDir": ".lake/packages",
"packages":
[{"url": "https://github.com/leanprover/std4",
[{"url": "https://github.com/leanprover-community/batteries",
"type": "git",
"subDir": null,
"rev": "3025cb124492b423070f20cf0a70636f757d117f",
"name": "std",
"rev": "56d2e4ee226603eb6b90b05f6b944bde42672cd5",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": false,
Expand Down
2 changes: 1 addition & 1 deletion lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ lean_lib ProofWidgets
lean_lib ProofWidgets.Demos where
globs := #[.submodules `ProofWidgets.Demos]

require std from git "https://github.com/leanprover/std4" @ "main"
require batteries from git "https://github.com/leanprover-community/batteries" @ "main"

def npmCmd : String :=
if Platform.isWindows then "npm.cmd" else "npm"
Expand Down

0 comments on commit e6b6247

Please sign in to comment.