src/Pure/Pure.thy
changeset 60957 574254152856
parent 60749 f727b99faaf7
child 61252 c165f0472d57
--- a/src/Pure/Pure.thy	Mon Aug 17 16:27:12 2015 +0200
+++ b/src/Pure/Pure.thy	Mon Aug 17 19:34:15 2015 +0200
@@ -21,7 +21,7 @@
     "definition" "abbreviation" "type_notation" "no_type_notation" "notation"
     "no_notation" "axiomatization" "theorems" "lemmas" "declare"
     "hide_class" "hide_type" "hide_const" "hide_fact" :: thy_decl
-  and "SML_file" :: thy_load % "ML"
+  and "SML_file" "SML_file_debug" "SML_file_no_debug" :: thy_load % "ML"
   and "SML_import" "SML_export" :: thy_decl % "ML"
   and "ML" :: thy_decl % "ML"
   and "ML_prf" :: prf_decl % "proof"  (* FIXME % "ML" ?? *)