lean2/tests/lean/584a.lean

19 lines
305 B
Text
Raw Normal View History

2015-05-07 21:24:30 +00:00
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:nat) := rfl
2015-05-07 21:24:30 +00:00
set_option pp.implicit true
print test