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

14 lines
288 B
Idris

parameters {n : Nat}
(a : Int)
0 func : Bool -> Type
func True = List Bool
func False = List Nat
getType : (b : Bool) -> func b
getType False = [0,1,2]
getType True = [True, True, True]
prf : (b : Bool) -> Int -> func b
prf b i = let i1 = getType b in ?whut