mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-16 07:34:45 +03:00
a972778eab
They don't all pass yet, for minor reasons. Coming shortly... Unfortunately the startup overhead for chez is really noticeable here!
14 lines
259 B
Idris
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
|