62408a6adc
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>
14 lines
259 B
Text
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
|