--- a/src/Tools/SML/Examples.thy Sun Jan 06 13:44:33 2019 +0100
+++ b/src/Tools/SML/Examples.thy Sun Jan 06 15:04:34 2019 +0100
@@ -21,7 +21,7 @@
evaluates it for some arguments.
\<close>
-SML_file "factorial.sml"
+SML_file \<open>factorial.sml\<close>
text \<open>
The subsequent example illustrates the use of multiple \<^theory_text>\<open>SML_file\<close> commands
@@ -30,8 +30,8 @@
independently of the Isabelle/ML environment.
\<close>
-SML_file "Example.sig"
-SML_file "Example.sml"
+SML_file \<open>Example.sig\<close>
+SML_file \<open>Example.sml\<close>
text \<open>