summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Arith/Int.lean
diff options
context:
space:
mode:
authorSon Ho2023-07-19 14:48:08 +0200
committerSon Ho2023-07-19 14:48:08 +0200
commit204742bf2449c88abaea8ebd284c55d98b43488a (patch)
tree2d554025cd8d8d88738e6bd24286d6eac2c239cc /backends/lean/Base/Arith/Int.lean
parent0a8211041814b5eafac0b9e2dbcd956957a322b5 (diff)
Improve progress
Diffstat (limited to '')
-rw-r--r--backends/lean/Base/Arith/Int.lean8
1 files changed, 0 insertions, 8 deletions
diff --git a/backends/lean/Base/Arith/Int.lean b/backends/lean/Base/Arith/Int.lean
index 5f00ab52..ac011998 100644
--- a/backends/lean/Base/Arith/Int.lean
+++ b/backends/lean/Base/Arith/Int.lean
@@ -32,14 +32,6 @@ instance (x y : Int) : PropHasImp (¬ x = y) where
open Lean Lean.Elab Lean.Meta
--- Small utility: print all the declarations in the context
-elab "print_all_decls" : tactic => do
- let ctx ← Lean.MonadLCtx.getLCtx
- for decl in ← ctx.getDecls do
- let ty ← Lean.Meta.inferType decl.toExpr
- logInfo m!"{decl.toExpr} : {ty}"
- pure ()
-
-- Explore a term by decomposing the applications (we explore the applied
-- functions and their arguments, but ignore lambdas, forall, etc. -
-- should we go inside?).