2014-07-07 21:41:14 +00:00
|
|
|
|
import standard
|
2014-08-15 20:27:18 +00:00
|
|
|
|
using prod
|
2014-07-07 21:41:14 +00:00
|
|
|
|
|
|
|
|
|
inductive t1 : Type :=
|
2014-08-22 22:46:10 +00:00
|
|
|
|
mk1 : t1
|
2014-07-07 21:41:14 +00:00
|
|
|
|
|
|
|
|
|
inductive t2 : Type :=
|
2014-08-22 22:46:10 +00:00
|
|
|
|
mk2 : t2
|
2014-07-07 21:41:14 +00:00
|
|
|
|
|
|
|
|
|
theorem inhabited_t1 : inhabited t1
|
2014-08-20 22:49:44 +00:00
|
|
|
|
:= inhabited_mk mk1
|
2014-07-07 21:41:14 +00:00
|
|
|
|
|
|
|
|
|
theorem inhabited_t2 : inhabited t2
|
2014-08-20 22:49:44 +00:00
|
|
|
|
:= inhabited_mk mk2
|
2014-07-07 21:41:14 +00:00
|
|
|
|
|
|
|
|
|
instance inhabited_t1 inhabited_t2
|
|
|
|
|
|
|
|
|
|
theorem T : inhabited (t1 × t2)
|
|
|
|
|
:= _
|