mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-25 12:42:02 +03:00
Add test files
This commit is contained in:
parent
ffbea6d160
commit
a52308d77d
16
tests/idris2/reg028/Test.idr
Normal file
16
tests/idris2/reg028/Test.idr
Normal 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
|
1
tests/idris2/reg028/expected
Normal file
1
tests/idris2/reg028/expected
Normal file
@ -0,0 +1 @@
|
||||
1/1: Building Test (Test.idr)
|
3
tests/idris2/reg028/run
Executable file
3
tests/idris2/reg028/run
Executable file
@ -0,0 +1,3 @@
|
||||
$1 --check Test.idr
|
||||
|
||||
rm -rf build
|
Loading…
Reference in New Issue
Block a user