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

5 lines
123 B
Idris

main : IO ()
main = do
putStrLn $ show (the Bits64 0xffffffffffffffff)
putStrLn $ show (the Bits64 0x8000000000000000)