src/Pure/ML_Bootstrap.thy
changeset 64331 abf7b6e6865f
parent 63220 06cbfbaf39c5
child 67105 05ff3e6dbbce
--- a/src/Pure/ML_Bootstrap.thy	Fri Oct 21 11:00:16 2016 +0200
+++ b/src/Pure/ML_Bootstrap.thy	Fri Oct 21 11:19:15 2016 +0200
@@ -15,7 +15,7 @@
 SML_import \<open>
   structure Output_Primitives = Output_Primitives_Virtual;
   structure Thread_Data = Thread_Data_Virtual;
-  fun ML_system_pp (_: int -> 'a -> 'b -> PolyML_Pretty.pretty) = ();
+  fun ML_system_pp (_: FixedInt.int -> 'a -> 'b -> PolyML_Pretty.pretty) = ();
 \<close>