summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Progress/Base.lean
diff options
context:
space:
mode:
authorSon Ho2023-12-11 18:34:10 +0100
committerSon Ho2023-12-11 18:34:10 +0100
commit78367ef21c147b26040e0f6062a907fceab1f390 (patch)
tree6dfb4095d4df161023164b512847ba90f3f72300 /backends/lean/Base/Progress/Base.lean
parentee669c4dbf8be12a3dd7249c645fd7092ba3e8eb (diff)
Start working on higher-order examples for Diverge
Diffstat (limited to 'backends/lean/Base/Progress/Base.lean')
-rw-r--r--backends/lean/Base/Progress/Base.lean6
1 files changed, 2 insertions, 4 deletions
diff --git a/backends/lean/Base/Progress/Base.lean b/backends/lean/Base/Progress/Base.lean
index fd80db8c..0ad16ab6 100644
--- a/backends/lean/Base/Progress/Base.lean
+++ b/backends/lean/Base/Progress/Base.lean
@@ -3,8 +3,6 @@ import Std.Lean.HashSet
import Base.Utils
import Base.Primitives.Base
import Base.Extensions
-import Lean.Meta.DiscrTree
-import Lean.Meta.Tactic.Simp
namespace Progress
@@ -101,7 +99,7 @@ section Methods
-- Check if some existentially quantified variables
let _ := do
-- Collect all the free variables in the arguments
- let allArgsFVars := ← args.foldlM (fun hs arg => getFVarIds arg hs) HashSet.empty
+ let allArgsFVars ← args.foldlM (fun hs arg => getFVarIds arg hs) HashSet.empty
-- Check if they intersect the fvars we introduced for the existentially quantified variables
let evarsSet : HashSet FVarId := HashSet.ofArray (evars.map (fun (x : Expr) => x.fvarId!))
let filtArgsFVars := allArgsFVars.toArray.filter (fun var => evarsSet.contains var)
@@ -134,7 +132,7 @@ structure PSpecAttr where
ext : DiscrTreeExtension Name true
deriving Inhabited
-/- The persistent map from function to pspec theorems. -/
+/- The persistent map from expressions to pspec theorems. -/
initialize pspecAttr : PSpecAttr ← do
let ext ← mkDiscrTreeExtention `pspecMap true
let attrImpl : AttributeImpl := {