summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Arith/Int.lean
diff options
context:
space:
mode:
authorSon Ho2024-04-05 14:04:25 +0200
committerSon Ho2024-04-05 14:04:25 +0200
commit65a77968d0abc2d01da92aa8982256855e7519a6 (patch)
tree5db0aaddd797ab769dcc72f46094fc6f3dc3b8a5 /backends/lean/Base/Arith/Int.lean
parentfc0b39c4fe48fdbab06d5fd32e0a2b7dcae674e6 (diff)
Update the lean toolchain and fix the proofs
Diffstat (limited to 'backends/lean/Base/Arith/Int.lean')
-rw-r--r--backends/lean/Base/Arith/Int.lean1
1 files changed, 0 insertions, 1 deletions
diff --git a/backends/lean/Base/Arith/Int.lean b/backends/lean/Base/Arith/Int.lean
index a57f8bb1..5a85dff0 100644
--- a/backends/lean/Base/Arith/Int.lean
+++ b/backends/lean/Base/Arith/Int.lean
@@ -3,7 +3,6 @@
import Lean
import Lean.Meta.Tactic.Simp
import Init.Data.List.Basic
-import Mathlib.Tactic.RunCmd
import Mathlib.Tactic.Linarith
-- TODO: there is no Omega tactic for now - it seems it hasn't been ported yet
--import Mathlib.Tactic.Omega