Idris2/tests/idris2/warning002/Main.idr
2021-11-17 10:41:03 +00:00

20 lines
317 B
Idris

module Main
import Foo
testConstValue1 : String
testConstValue1 = dep1
testConstValue2 : String
testConstValue2 = dep2
testFunctionPass : String -> String
testFunctionPass = dep3
testErasedFunction : List Int -> Foo.foo Int
testErasedFunction xs = xs
0 testInErasedContext : Type
testInErasedContext = foo Int