Idris2/tests/idris2/literate/literate007/IEdit.org
2023-09-07 14:57:22 +01:00

329 B

data Vect : Nat -> Type -> Type where
     Nil : Vect Z a
     (::) : a -> Vect k a -> Vect (S k) a