8de9cab62d
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
9 lines
189 B
Text
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
|