mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
8 lines
167 B
Idris
8 lines
167 B
Idris
|
import Data.Vect
|
||
|
|
||
|
data VectN : Type -> Type where
|
||
|
MkVectN : (n : Nat) -> Vect n a -> VectN a
|
||
|
|
||
|
doSearch : Nat -> VectN Int
|
||
|
doSearch n = MkVectN ?vlength [1,2,3,4]
|