9 lines
190 B
Text
9 lines
190 B
Text
import logic data.prod data.num
|
||
open prod nonempty inhabited
|
||
|
||
theorem H {A B : Type} (H1 : inhabited A) : inhabited (Prop × A × (B → num))
|
||
:= _
|
||
|
||
(*
|
||
print(get_env():find("H"):value())
|
||
*)
|