Idris2/tests/idris2/misc/import009/Prefix.idr
2023-09-07 14:57:22 +01:00

13 lines
150 B
Idris

module Prefix
private
prefix 5 !!
export
(!!) : Type -> Type
(!!) = Not
export
test : Either (!! a) (!! b) -> !! (a, b)
test f (x, y) = f (Left x)