lean2/tests/lean/run/ind2.lean
Leonardo de Moura a5f0593df1 feat(*): change inductive datatype syntax
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-22 15:46:10 -07:00

12 lines
258 B
Text

inductive nat : Type :=
zero : nat,
succ : nat → nat
inductive vector (A : Type) : nat → Type :=
vnil : vector A zero,
vcons : Π {n : nat}, A → vector A n → vector A (succ n)
check vector.{1}
check vnil.{1}
check vcons.{1}
check vector_rec.{1 1}