lean2/tests/lean/run/class3.lean

18 lines
269 B
Text
Raw Normal View History

import logic data.prod
open prod inhabited
section
variable {A : Type}
variable {B : Type}
variable Ha : inhabited A
variable Hb : inhabited B
include Ha Hb
theorem tst : inhabited (Prop × A × B)
end
wait tst
(*
print(get_env():find("tst"):value())
*)