lean2/tests/lean/run/t11.lean
2014-10-09 07:13:06 -07:00

14 lines
266 B
Text

constant A : Type.{1}
constants a b c : A
constant f : A → A → A
check f a b
context
parameters A B : Type
parameters {C D : Type}
parameters [e d : A]
check A
check B
definition g (a : A) (b : B) (c : C) : A := e
end
check g.{2 1}
constants x y : A