lean2/tests/lean/rw_set2.lean

13 lines
200 B
Text
Raw Permalink Normal View History

open nat
constant f : nat → nat
constant g : nat → nat
axiom foo : ∀ x, x > 0 → f x = 0 ∧ g x = 1
axiom bla : ∀ x, g x = f x + 1
attribute foo [simp]
attribute bla [simp]
print [simp]