Idris2/tests/idris2/interactive/interactive015/IEdit.idr
2023-09-07 14:57:22 +01:00

18 lines
440 B
Idris

data Vect : Nat -> Type -> Type where
Nil : Vect Z a
(::) : a -> Vect k a -> Vect (S k) a
%name Vect xs, ys, zs
my_cong : forall f . (x : a) -> (y : a) -> x = y -> f x = f y
append : Vect n a -> Vect m a -> Vect (n + m) a
lappend : (1 _ : List a) -> (1 _ : List a) -> List a
lappend1 : List a -> List a -> List a
lappend2 : List a -> List a -> List a
lappend2 [] ys = ?lappend2_rhs_1
lappend2 (x :: xs) ys = ?lappend2_rhs_2