Skip to content

Commit

Permalink
Merge pull request #26 from dranov/bump-v4.11.0
Browse files Browse the repository at this point in the history
Bump to v4.11.0
  • Loading branch information
JOSHCLUNE authored Oct 3, 2024
2 parents f4c5e9b + 9f6b4b3 commit 04377f4
Show file tree
Hide file tree
Showing 6 changed files with 10 additions and 11 deletions.
1 change: 0 additions & 1 deletion Duper/Preprocessing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,6 @@ namespace Duper
namespace ProverM
open Lean
open Meta
open Std
open ProverM
open RuleM
open SimpResult
Expand Down
1 change: 0 additions & 1 deletion Duper/ProverM.lean
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,6 @@ namespace Duper
namespace ProverM
open Lean
open Lean.Core
open Std
open RuleM
open Expr

Expand Down
1 change: 0 additions & 1 deletion Duper/SubsumptionTrie.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ namespace Duper

open Lean
open RuleM
open Std
open List
open Expr

Expand Down
12 changes: 7 additions & 5 deletions lake-manifest.json
Original file line number Diff line number Diff line change
@@ -1,22 +1,24 @@
{"version": "1.0.0",
{"version": "1.1.0",
"packagesDir": ".lake/packages",
"packages":
[{"url": "https://github.com/leanprover-community/lean-auto.git",
"type": "git",
"subDir": null,
"rev": "1ba441f1d385cc2a7eebd927a5d2aa71b40fbd7a",
"scope": "",
"rev": "bfd373fb8ee85a0255f64b4f376e5fb08bb8a1da",
"name": "auto",
"manifestFile": "lake-manifest.json",
"inputRev": "1ba441f1d385cc2a7eebd927a5d2aa71b40fbd7a",
"inputRev": "v4.11.0",
"inherited": false,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/batteries",
"type": "git",
"subDir": null,
"rev": "dcea9ce8aba248927fb2ea8d5752bfe1e3fe7b44",
"scope": "",
"rev": "9c6c2d647e57b2b7a0b42dd8080c698bd33a1b6f",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.9.1",
"inputRev": "v4.11.0",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "Duper",
Expand Down
4 changes: 2 additions & 2 deletions lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,8 +2,8 @@ import Lake

open Lake DSL

require auto from git "https://github.com/leanprover-community/lean-auto.git"@"1ba441f1d385cc2a7eebd927a5d2aa71b40fbd7a"
require batteries from git "https://github.com/leanprover-community/batteries" @ "v4.9.1"
require auto from git "https://github.com/leanprover-community/lean-auto.git"@"v4.11.0"
require batteries from git "https://github.com/leanprover-community/batteries" @ "v4.11.0"

package Duper {
precompileModules := true
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.9.1
leanprover/lean4:v4.11.0

0 comments on commit 04377f4

Please sign in to comment.