Idris2/tests/idris2/error/perror021/Implicit.idr
2023-09-07 14:57:22 +01:00

7 lines
179 B
Idris

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])