16 lines
260 B
Text
16 lines
260 B
Text
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
|
||
|
||
(*
|
||
print(get_env():find("tst"):value())
|
||
*)
|