Skip to content

Commit fd52edd

Browse files
committed
workaround for tests?
1 parent 4da773a commit fd52edd

File tree

3 files changed

+6
-0
lines changed

3 files changed

+6
-0
lines changed

tests/lean/run/list_simp.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,5 @@
1+
import Lean.Elab.CheckTactic
2+
13
set_option autoImplicit false -- For compatibility with downstream projects, so we can retest after Mathlib.
24
set_option relaxedAutoImplicit false
35

tests/lean/run/simprocNat.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,5 @@
1+
import Lean.Elab.CheckTactic
2+
13
variable (a b : Nat)
24

35
/- bitwise operation tests -/

tests/lean/simpArrayIdx.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,5 @@
1+
import Lean.Elab.CheckTactic
2+
13
section
24
variable {α : Type _}
35
variable [Inhabited α]

0 commit comments

Comments
 (0)