lean2/tests/lean/slow/simp_loop.lean
Leonardo de Moura 62408a6adc test(tests/lean): move simp_loop test to slow subdirectory
This example produces a stackoverflow on Valgrind.
We don't execute Valgrind on tests in the slow subdirectory.

Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-29 10:32:48 -08:00

14 lines
259 B
Text

import tactic
import macros
variable f : Nat → Nat
variable g : Nat → Nat
axiom Ax1 (a : Nat) : f a = g a
axiom Ax2 (a : Nat) : g a = f a
add_rewrite Ax1 Ax2
-- The following call to simp should produce a stack overflow
theorem T : f 0 = 0
:= by simp