lean2/tests/lean/interactive/simple3.lean
Leonardo de Moura 8de9cab62d test(tests/lean/interactive): add --server test
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-28 07:41:38 -07:00

9 lines
189 B
Text

import logic
namespace tst
definition foo {A B : Type} (a : A) (b : B) := a
definition boo {A : Type} (a : A) := foo a a
end tst
theorem tst {A : Type} (a b : A) : tst.foo a b = a :=
rfl