src/ZF/Inductive.thy
changeset 69605 a96320074298
parent 69597 ff784d5a5bfb
child 74296 abc878973216
--- a/src/ZF/Inductive.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/ZF/Inductive.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -27,12 +27,12 @@
 
 lemma refl_thin: "!!P. a = a ==> P ==> P" .
 
-ML_file "ind_syntax.ML"
-ML_file "Tools/ind_cases.ML"
-ML_file "Tools/cartprod.ML"
-ML_file "Tools/inductive_package.ML"
-ML_file "Tools/induct_tacs.ML"
-ML_file "Tools/primrec_package.ML"
+ML_file \<open>ind_syntax.ML\<close>
+ML_file \<open>Tools/ind_cases.ML\<close>
+ML_file \<open>Tools/cartprod.ML\<close>
+ML_file \<open>Tools/inductive_package.ML\<close>
+ML_file \<open>Tools/induct_tacs.ML\<close>
+ML_file \<open>Tools/primrec_package.ML\<close>
 
 ML \<open>
 structure Lfp =