src/FOLP/IFOLP.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 70880 de2e2382bc0d
--- a/src/FOLP/IFOLP.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/FOLP/IFOLP.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -9,7 +9,7 @@
 imports Pure
 begin
 
-ML_file "~~/src/Tools/misc_legacy.ML"
+ML_file \<open>~~/src/Tools/misc_legacy.ML\<close>
 
 setup Pure_Thy.old_appl_syntax_setup
 
@@ -605,7 +605,7 @@
 
 lemma thin_refl: "!!X. [|p:x=x; PROP W|] ==> PROP W" .
 
-ML_file "hypsubst.ML"
+ML_file \<open>hypsubst.ML\<close>
 
 ML \<open>
 structure Hypsubst = Hypsubst
@@ -627,7 +627,7 @@
 open Hypsubst;
 \<close>
 
-ML_file "intprover.ML"
+ML_file \<open>intprover.ML\<close>
 
 
 (*** Rewrite rules ***)