Add test files

This commit is contained in:
Edwin Brady 2020-06-29 15:13:42 +01:00
parent ffbea6d160
commit a52308d77d
3 changed files with 20 additions and 0 deletions

View File

@ -0,0 +1,16 @@
module Test
data Dummy : (lbl : Type) -> (st : List lbl) -> Type -> Type where
MkDummy : a -> Dummy b st a
public export
interface IxPure (f : (lbl : Type) -> (st : List lbl) -> Type -> Type)
where
ixPure : a -> f lbl st a
IxPure Dummy where
ixPure = MkDummy
pure12 : Dummy String xs Nat
pure12 = ixPure Z

View File

@ -0,0 +1 @@
1/1: Building Test (Test.idr)

3
tests/idris2/reg028/run Executable file
View File

@ -0,0 +1,3 @@
$1 --check Test.idr
rm -rf build