add tests to chaining and combing operators

This commit is contained in:
André Videla 2023-10-22 13:42:13 +01:00
parent 6ce4ec2ebf
commit 1adb780e3f

View File

@ -3,13 +3,20 @@
import Data.Vect
typebind infixr 0 =@
infixr 0 -@
0 (=@) : (a : Type) -> (a -> Type) -> Type
(=@) a f = (1 x : a) -> f x
(-@) : (a, b : Type) -> Type
(-@) a b = (1 _ : a) -> b
data S : {ty : Type} -> (x : ty) -> Type where
MkS : (x : ty) =@ S x
Mk2 : (x : ty) =@ (y : ty) =@ S (x, y)
Mk3 : (x : ty) =@ ty -@ S x
Mk4 : ty -@ (x : ty) =@ S x
-- Chain : (x : ty =@ y : ty =@ S (x, y))
typebind infixr 0 *>