We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent ae7b5f0 commit e1524ddCopy full SHA for e1524dd
tests/idris2/linear/linear019/Issue490.idr
@@ -0,0 +1,7 @@
1
+data MyList : Type -> Type where
2
+ Nil : {a : Type} -> MyList a
3
+ (::) : {a : Type} -> a -> MyList a -> MyList a
4
+
5
+g : MyList a -> ()
6
+g [] = ()
7
+g l@(x :: xs) = ?hole
tests/idris2/linear/linear019/expected
@@ -0,0 +1,9 @@
+1/1: Building Issue490 (Issue490.idr)
+Main> a : Type
+ x : a
+ xs : MyList a
+ l : MyList a
+------------------------------
+hole : ()
8
+Main>
9
+Bye for now!
tests/idris2/linear/linear019/input
@@ -0,0 +1 @@
+:t hole
tests/idris2/linear/linear019/run
@@ -0,0 +1,3 @@
+. ../../../testutils.sh
+idris2 Issue490.idr < input
0 commit comments