lean2/tests/lean/sec_param_pp.lean
2015-04-21 22:44:09 -07:00

20 lines
271 B
Text

section
parameters {A : Type} (a : A)
variable f : A → A → A
definition id : A := a
check id
definition pr (b : A) : A := f a b
check pr f id
set_option pp.universes true
check pr f id
definition pr2 (B : Type) (b : B) : A := a
check pr2 num 10
end