Idris2/tests/idris2/error/perror021/Implicit.idr

7 lines
179 B
Idris
Raw Normal View History

import Data.Vect
myReverse : Vect n el -> Vect n el
myReverse [] = []
myReverse {n = S k} (x :: xs) =
replace {p=\n => Vect n el} (plusCommutative k 1) (myReverse xs ++ [x])