mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-16 07:34:45 +03:00
15 lines
291 B
Idris
15 lines
291 B
Idris
|
|
module NoRegression
|
|
|
|
import Data.Vect
|
|
|
|
data Dep : (n : Nat) -> (a : Type) -> Vect n a -> Type where
|
|
MkDep : Dep n a v
|
|
|
|
dpairParse : ( n : Nat
|
|
** a : Type
|
|
** v : Vect n a
|
|
** Dep n a v
|
|
)
|
|
dpairParse = (_ ** _ ** ["a", "b"] ** MkDep)
|