Skip to content

Commit

Permalink
Update to lean v4.11.0
Browse files Browse the repository at this point in the history
  • Loading branch information
JOSHCLUNE committed Oct 13, 2024
2 parents 92c1afd + ad292bd commit 87d7f13
Show file tree
Hide file tree
Showing 7 changed files with 11 additions and 12 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
2 changes: 1 addition & 1 deletion README.md
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ Duper is an automatic proof-producing theorem prover broadly similar to Isabelle
To use Duper in an existing Lean 4 project, first add this package as a dependency. In your lakefile.lean, add:

```lean
require Duper from git "https://github.com/leanprover-community/duper.git" @ "v0.0.15"
require Duper from git "https://github.com/leanprover-community/duper.git" @ "v0.0.16"
```

Then, make sure that your `lean-toolchain` file contains the same version of Lean 4 as Duper and that if your project imports [batteries](https://github.com/leanprover-community/batteries), then it uses the same version of batteries as Duper. This step is necessary because Duper depends on batteries, so errors can arise if your project attempts to import a version of batteries different from the one imported by Duper.
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": "22d4c2e7f2453e16b9d980cae2367d38bedf3bf5",
"scope": "",
"rev": "2b6ed7d9f86d558d94b8d9036a637395163c4fa6",
"name": "auto",
"manifestFile": "lake-manifest.json",
"inputRev": "22d4c2e7f2453e16b9d980cae2367d38bedf3bf5",
"inputRev": "2b6ed7d9f86d558d94b8d9036a637395163c4fa6",
"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"@"22d4c2e7f2453e16b9d980cae2367d38bedf3bf5"
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"@"2b6ed7d9f86d558d94b8d9036a637395163c4fa6"
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 87d7f13

Please sign in to comment.