src/HOL/Nonstandard_Analysis/StarDef.thy
changeset 69605 a96320074298
parent 69597 ff784d5a5bfb
child 69700 7a92cbec7030
--- a/src/HOL/Nonstandard_Analysis/StarDef.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/HOL/Nonstandard_Analysis/StarDef.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -99,7 +99,7 @@
   where "star_of x \<equiv> star_n (\<lambda>n. x)"
 
 text \<open>Initialize transfer tactic.\<close>
-ML_file "transfer_principle.ML"
+ML_file \<open>transfer_principle.ML\<close>
 
 method_setup transfer =
   \<open>Attrib.thms >> (fn ths => fn ctxt => SIMPLE_METHOD' (Transfer_Principle.transfer_tac ctxt ths))\<close>