summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Utils.lean
diff options
context:
space:
mode:
authorSon HO2023-09-14 08:19:59 +0200
committerGitHub2023-09-14 08:19:59 +0200
commit242aca3092c6594206896ea62eb40395accc8459 (patch)
tree4a105b1284821a89ca344188fdddb727de2deea3 /backends/lean/Base/Utils.lean
parentda97fc1e68d147439436ff883ac865a9cdeca18e (diff)
parent743e8cb9d5366b879f53d7d0ba8adeb2f83ef72f (diff)
Merge pull request #36 from AeneasVerif/update_lean
Update the version of Lean and fix a bug in the progress tactic
Diffstat (limited to 'backends/lean/Base/Utils.lean')
-rw-r--r--backends/lean/Base/Utils.lean4
1 files changed, 4 insertions, 0 deletions
diff --git a/backends/lean/Base/Utils.lean b/backends/lean/Base/Utils.lean
index 1f8f1455..5224e1c3 100644
--- a/backends/lean/Base/Utils.lean
+++ b/backends/lean/Base/Utils.lean
@@ -301,6 +301,10 @@ example : Nat := by
example (x : Bool) : Nat := by
cases x <;> custom_let x := 3 <;> apply x
+-- Attempt to apply a tactic
+def tryTac (tac : TacticM Unit) : TacticM Unit := do
+ let _ ← tryTactic tac
+
-- Repeatedly apply a tactic
partial def repeatTac (tac : TacticM Unit) : TacticM Unit := do
try