Skip to content

Commit

Permalink
rm open private
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Oct 16, 2024
1 parent 88169a8 commit 6503af8
Show file tree
Hide file tree
Showing 4 changed files with 4 additions and 6 deletions.
2 changes: 0 additions & 2 deletions Aesop/Util/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -29,8 +29,6 @@ def replaceFVar (goal : MVarId) (fvarId : FVarId) (type : Expr) (proof : Expr) :
let (newFVarId, goal) ← intro1Core goal (preserveBinderNames := true)
return (goal, newFVarId, clearSuccess)

open private getIntrosSize in Lean.MVarId.intros

/-- Introduce as many binders as possible while unfolding definitions with the
ambient transparency. -/
partial def introsUnfolding (mvarId : MVarId) : MetaM (Array FVarId × MVarId) :=
Expand Down
4 changes: 2 additions & 2 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,10 +5,10 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "fc871f7039ac6d8ab993335bb35aba43286004a0",
"rev": "0a6bfc711cbc3b4a98d89a65bc904c361a792386",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inputRev": "nightly-testing",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "aesop",
Expand Down
2 changes: 1 addition & 1 deletion lakefile.toml
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ precompileModules = false # We would like to turn this on, but it breaks the Mat
[[require]]
name = "batteries"
git = "https://github.com/leanprover-community/batteries"
rev = "main"
rev = "nightly-testing"

[[lean_lib]]
name = "Aesop"
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.13.0-rc1
leanprover/lean4:nightly-2024-10-16

0 comments on commit 6503af8

Please sign in to comment.