Idris2/tests/idris2/basic/basic066/comment.idr
2023-09-07 14:57:22 +01:00

13 lines
241 B
Idris

{--- -}
fun : Int -> Bool
fun x = (x /= 0)
{-
-}
main : IO ()
main = print (fun 5)
-- EXPLANATION:
-- this is about parsing the opening `{---`
-- which used to be parsed as two separate tokens `{-` and `--`
-- making the above program fail