lean2/tests/lean/771.lean
Leonardo de Moura 5568085ab9 fix(frontends/lean/elaborator): closes #771
Produce nicer error message when type/goal is a metavariable and
universe metavariables have already been instantiated with universe
parameters.
2015-08-07 13:29:22 -07:00

12 lines
216 B
Text

set_option pp.all true
definition id_1 (n : nat) :=
by exact n
definition id_2 (n : nat) :=
(by exact n : nat)
definition id_3 (n : nat) : nat :=
by exact n
definition id_4 (n : nat) :=
show nat, by exact n