mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
10 lines
169 B
Idris
10 lines
169 B
Idris
module Import
|
|
|
|
import Test
|
|
|
|
(|>) : (s : HasComp x) => {0 a, b, c : x} -> a ~> b -> b ~> c -> a ~> c
|
|
a |> b = comp s a b
|
|
|
|
(~:>) : Type -> Type -> Type
|
|
a ~:> b = Pair a b
|