diff -r 51fdede038c9 -r 10732941cc4b src/Pure/ML_Bootstrap.thy --- a/src/Pure/ML_Bootstrap.thy Sat Aug 25 22:14:12 2018 +0200 +++ b/src/Pure/ML_Bootstrap.thy Sun Aug 26 15:39:34 2018 +0200 @@ -26,16 +26,13 @@ ML \Proofterm.proofs := 0\ -ML \ - Context.setmp_generic_context NONE - ML \ - List.app ML_Name_Space.forget_structure ML_Name_Space.hidden_structures; - structure PolyML = - struct - val pointerEq = pointer_eq; - structure IntInf = PolyML.IntInf; - end; - \ +ML_export \ + List.app ML_Name_Space.forget_structure ML_Name_Space.hidden_structures; + structure PolyML = + struct + val pointerEq = pointer_eq; + structure IntInf = PolyML.IntInf; + end; \ ML \\<^assert> (not (can ML \open RunCall\))\