mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 01:01:59 +03:00
11 lines
253 B
Idris
11 lines
253 B
Idris
test : {a : Nat} -> (b : Nat) -> a === b -> Nat
|
|
test a eq = ?a
|
|
|
|
data Vect : Nat -> Type -> Type where
|
|
Nil : Vect 0 a
|
|
(::) : a -> Vect n a -> Vect (S n) a
|
|
|
|
append : Vect n a -> Vect m a -> Vect (n + m) a
|
|
append [] ys = ys
|
|
append (x :: xs) ys = ?help
|