lean2/tests/lean/584a.lean
2015-05-07 14:24:30 -07:00

18 lines
299 B
Text

variables (A : Type) [H : inhabited A] (x : A)
include H
definition foo := x
check foo -- A and x are explicit
variables {A x}
definition foo' := x
check @foo' -- A is explicit, x is implicit
open nat
check foo nat 10
definition test : foo' = 10 := rfl
set_option pp.implicit true
print test