mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-30 07:02:24 +03:00
12 lines
333 B
Idris
12 lines
333 B
Idris
|
import System
|
||
|
|
||
|
main : IO ()
|
||
|
main = do
|
||
|
0 <- system "bash zero.sh"
|
||
|
| r => do putStrLn ("expecting zero, got " ++ (show r))
|
||
|
exitFailure
|
||
|
-- `system` returns result of `waitpid` which is not trivial to decode
|
||
|
let True = !(system "bash seventeen.sh") /= 0
|
||
|
| False => putStrLn "expecting 17, got zero"
|
||
|
pure ()
|