lean2/tests/lean/simp33.lean
Leonardo de Moura c56df132b8 refactor(kernel): remove semantic attachments from the kernel
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-02-02 14:48:27 -08:00

9 lines
229 B
Text

import tactic
variable f {A : TypeU} : A → A
axiom Ax1 (a : Bool) : f a = not a
axiom Ax2 (a : Nat) : f a = 0
rewrite_set S
add_rewrite Ax1 Ax2 not_false : S
theorem T1 (a : Nat) : f (f a > 0)
:= by simp S
print environment 1