summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Arith/Int.lean
diff options
context:
space:
mode:
authorSon Ho2023-09-14 07:07:44 +0200
committerSon Ho2023-09-14 07:07:44 +0200
commit0504acdaee98f28dfd08c5652b39c201c252d1be (patch)
tree0ba96dd2a488e0cb98442ad67030f0e637b9670b /backends/lean/Base/Arith/Int.lean
parentda97fc1e68d147439436ff883ac865a9cdeca18e (diff)
Update to Lean 4.0.0 and fix some broken proofs
Diffstat (limited to '')
-rw-r--r--backends/lean/Base/Arith/Int.lean2
1 files changed, 1 insertions, 1 deletions
diff --git a/backends/lean/Base/Arith/Int.lean b/backends/lean/Base/Arith/Int.lean
index 531ec94f..eb6701c2 100644
--- a/backends/lean/Base/Arith/Int.lean
+++ b/backends/lean/Base/Arith/Int.lean
@@ -238,7 +238,7 @@ def intTac (splitGoalConjs : Bool) (extraPreprocess : Tactic.TacticM Unit) : Ta
-- the goal. I think before leads to a smaller proof term?
Tactic.allGoals (intTacPreprocess extraPreprocess)
-- More preprocessing
- Tactic.allGoals (Utils.simpAt [] [``nat_zero_eq_int_zero] [] .wildcard)
+ Tactic.allGoals (Utils.tryTac (Utils.simpAt [] [``nat_zero_eq_int_zero] [] .wildcard))
-- Split the conjunctions in the goal
if splitGoalConjs then Tactic.allGoals (Utils.repeatTac Utils.splitConjTarget)
-- Call linarith