Idris2/tests/idris2/reg003/Holes.idr
Edwin Brady a972778eab Add test script
They don't all pass yet, for minor reasons. Coming shortly...
Unfortunately the startup overhead for chez is really noticeable here!
2020-05-19 18:25:18 +01:00

14 lines
259 B
Idris

import Data.Vect
import Data.Fin
Vect_ext : (v : Vect n a) -> (w : Vect n a) -> ((i : Fin n) -> index i v = index i w)
-> v = w
Weird : (v: Vect n a) -> v = v
Weird v = Vect_ext ?hole0 ?hole1 ?hole2
f : Bool -> Nat
f True = 0
f True = ?help
f False = 1