Idris2/tests/idris2/warning002/Foo.idr

24 lines
293 B
Idris
Raw Normal View History

2021-11-17 13:41:03 +03:00
module Foo
%deprecate
export
dep1 : String
dep1 = "hello"
||| Just use the string "world" directly from now on.
%deprecate
export
dep2 : String
dep2 = "world"
%deprecate
export
dep3 : String -> String
dep3 x = x ++ "!"
%deprecate
public export
0 foo : (0 a : Type) -> Type
foo x = List x