summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Arith/Int.lean
diff options
context:
space:
mode:
authorSon Ho2023-07-20 14:14:34 +0200
committerSon Ho2023-07-20 14:14:34 +0200
commit03492250b45855fe9db5e0a28a96166607cd84a1 (patch)
tree6ea4a188d630cf2d25704f09d6dc301aa6576a09 /backends/lean/Base/Arith/Int.lean
parent6ef1d360b89fd9f9383e63609888bf925a6a16ab (diff)
Make some proofs in Hashmap/Properties.lean and improve progress
Diffstat (limited to 'backends/lean/Base/Arith/Int.lean')
-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 ac011998..fa957293 100644
--- a/backends/lean/Base/Arith/Int.lean
+++ b/backends/lean/Base/Arith/Int.lean
@@ -198,7 +198,7 @@ def intTac (extraPreprocess : Tactic.TacticM Unit) : Tactic.TacticM Unit := do
-- Split the conjunctions in the goal
Tactic.allGoals (Utils.repeatTac Utils.splitConjTarget)
-- Call linarith
- let linarith :=
+ let linarith := do
let cfg : Linarith.LinarithConfig := {
-- We do this with our custom preprocessing
splitNe := false