Theory Native_Word_Test_PolyML64

(*  Title:      Native_Word_Test_PolYML64.thy
    Author:     Andreas Lochbihler, ETH Zurich
*)

theory Native_Word_Test_PolyML64 imports
  Native_Word_Test
begin

test_code "test_uint64' = 0x12"
in PolyML

ML if ML_System.platform_is_64 then
    ML assert (code‹test_uint64'› = 0wx12)›
  else ()

end