lean2/tests/lean/simp10.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

20 lines
No EOL
359 B
Text

variable f : Nat → Nat
variable g : Nat → Nat
variable a : Nat
axiom fid (x : Nat) : g x ≠ 0 → f x = x
add_rewrite fid
axiom gcnst (x : Nat) : g x = 1
add_rewrite gcnst
theorem one_neq_0 : 1 ≠ 0
:= Nat::succ_nz 0
add_rewrite one_neq_0
(*
local t = parse_lean("f a")
local r, pr = simplify(t)
print(r)
print(pr)
get_environment():type_check(pr)
*)