Idris2/tests/idris2/error/perror011/Issue1496-1.idr
2023-09-07 14:57:22 +01:00

9 lines
103 B
Idris

module Main
export
Show Really where
show (Really err) = ["RR"
main : IO ()
main = putStrLn "LOG"