mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 16:21:46 +03:00
14 lines
288 B
Idris
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
|
||
|
|