5568085ab9
Produce nicer error message when type/goal is a metavariable and universe metavariables have already been instantiated with universe parameters.
12 lines
216 B
Text
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
|