lean2/tests/lean/run/record6.lean
Leonardo de Moura b6722a5d33 feat(frontends/lean/structure_cmd): add 'private' modifier for parent structures
When it is used coercions/instances to parent structure are to registered
2014-11-03 23:16:49 -08:00

14 lines
308 B
Text

import logic data.unit
structure point (A : Type) (B : Type) :=
mk :: (x : A) (y : B)
structure point2 (A : Type) (B : Type) extends point A B :=
make
structure point3 extends point num num, private point2 num num renaming x→y y→z
check point3.mk
theorem tst : point3.mk 1 2 3 = point.mk 1 2 :=
rfl