mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-20 18:21:47 +03:00
24 lines
293 B
Idris
24 lines
293 B
Idris
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
|
|
|