Idris2/tests/idris2/perf005/NoRegression.idr

15 lines
291 B
Idris
Raw Normal View History

2020-09-05 12:03:35 +03:00
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)