diff -r a594429637fd -r fdd6989cc8a0 src/Doc/Implementation/ML.thy --- a/src/Doc/Implementation/ML.thy Wed Feb 17 21:08:18 2016 +0100 +++ b/src/Doc/Implementation/ML.thy Wed Feb 17 23:06:24 2016 +0100 @@ -505,7 +505,7 @@ ML and Isar are intertwined via an open-ended bootstrap process that provides more and more programming facilities and logical content in an alternating manner. Bootstrapping starts from the raw environment of - existing implementations of Standard ML (mainly Poly/ML, but also SML/NJ). + existing implementations of Standard ML (mainly Poly/ML). Isabelle/Pure marks the point where the raw ML toplevel is superseded by Isabelle/ML within the Isar theory and proof language, with a uniform @@ -1379,8 +1379,7 @@ \<^descr> Type @{ML_type int} represents regular mathematical integers, which are \<^emph>\unbounded\. Overflow is treated properly, but should never happen in practice.\<^footnote>\The size limit for integer bit patterns in memory is 64\,MB for - 32-bit Poly/ML, and much higher for 64-bit systems.\ This works uniformly - for all supported ML platforms (Poly/ML and SML/NJ). + 32-bit Poly/ML, and much higher for 64-bit systems.\ Literal integers in ML text are forced to be of this one true integer type --- adhoc overloading of SML97 is disabled.