lean2/tests/lean/run/class2.lean

9 lines
154 B
Text
Raw Normal View History

import standard
using num
theorem H {A B : Type} (H1 : inhabited A) : inhabited (Bool × A × (B → num))
:= _
(*
print(get_env():find("H"):value())
*)