2014-08-24 19:58:48 -07:00
|
|
|
|
import logic data.prod
|
2014-09-03 16:00:38 -07:00
|
|
|
|
open prod
|
2014-07-07 14:41:14 -07:00
|
|
|
|
|
|
|
|
|
inductive t1 : Type :=
|
2014-08-22 15:46:10 -07:00
|
|
|
|
mk1 : t1
|
2014-07-07 14:41:14 -07:00
|
|
|
|
|
|
|
|
|
inductive t2 : Type :=
|
2014-08-22 15:46:10 -07:00
|
|
|
|
mk2 : t2
|
2014-07-07 14:41:14 -07:00
|
|
|
|
|
|
|
|
|
theorem inhabited_t1 : inhabited t1
|
2014-09-04 16:36:06 -07:00
|
|
|
|
:= inhabited.mk t1.mk1
|
2014-07-07 14:41:14 -07:00
|
|
|
|
|
|
|
|
|
theorem inhabited_t2 : inhabited t2
|
2014-09-04 16:36:06 -07:00
|
|
|
|
:= inhabited.mk t2.mk2
|
2014-07-07 14:41:14 -07:00
|
|
|
|
|
|
|
|
|
instance inhabited_t1 inhabited_t2
|
|
|
|
|
|
|
|
|
|
theorem T : inhabited (t1 × t2)
|
|
|
|
|
:= _
|