2014-11-04 01:39:52 +00:00
|
|
|
import logic data.sigma
|
|
|
|
|
|
|
|
inductive point (A B : Type) :=
|
|
|
|
mk : Π (x : A) (y : B), point A B
|
|
|
|
|
|
|
|
inductive color [class] :=
|
2015-02-26 01:00:10 +00:00
|
|
|
red | green | blue
|
2014-11-04 01:39:52 +00:00
|
|
|
|
|
|
|
constant foo.{l} (A : Type.{l}) [H : decidable_eq A] : Type.{l}
|
|
|
|
|
|
|
|
constants a : num
|
|
|
|
|
|
|
|
section
|
|
|
|
universe variable l
|
|
|
|
variable A : Type.{l}
|
|
|
|
variable Ha : decidable_eq A
|
2015-02-20 06:43:28 +00:00
|
|
|
include Ha
|
2014-11-04 01:39:52 +00:00
|
|
|
variable E : Type₂
|
|
|
|
include E
|
|
|
|
-- include Ha
|
|
|
|
|
2014-12-20 02:23:08 +00:00
|
|
|
structure point3d_color (B C : Type) (D : B → Type) extends point (foo A) B, sigma D renaming pr1→y pr2→w :=
|
2014-11-04 01:39:52 +00:00
|
|
|
mk :: (c : color) (H : x == y)
|
|
|
|
|
|
|
|
check point3d_color.c
|
|
|
|
|
|
|
|
check point3d_color.to_point
|
|
|
|
end
|
|
|
|
|
2015-04-22 02:33:21 +00:00
|
|
|
section
|
2014-11-04 01:39:52 +00:00
|
|
|
universe l
|
|
|
|
parameters A : Type.{l}
|
|
|
|
parameters B : Type.{l}
|
|
|
|
|
|
|
|
structure tst :=
|
|
|
|
mk :: (a : A) (b : B)
|
|
|
|
|
|
|
|
end
|