src/CTT/CTT.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 74299 16e5870fe21e
--- a/src/CTT/CTT.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/CTT/CTT.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -9,7 +9,7 @@
 
 section \<open>Constructive Type Theory: axiomatic basis\<close>
 
-ML_file "~~/src/Provers/typedsimp.ML"
+ML_file \<open>~~/src/Provers/typedsimp.ML\<close>
 setup Pure_Thy.old_appl_syntax_setup
 
 typedecl i
@@ -455,7 +455,7 @@
 method_setup pc = \<open>Attrib.thms >> (fn ths => fn ctxt => SIMPLE_METHOD' (pc_tac ctxt ths))\<close>
 method_setup add_mp = \<open>Scan.succeed (SIMPLE_METHOD' o add_mp_tac)\<close>
 
-ML_file "rew.ML"
+ML_file \<open>rew.ML\<close>
 method_setup rew = \<open>Attrib.thms >> (fn ths => fn ctxt => SIMPLE_METHOD (rew_tac ctxt ths))\<close>
 method_setup hyp_rew = \<open>Attrib.thms >> (fn ths => fn ctxt => SIMPLE_METHOD (hyp_rew_tac ctxt ths))\<close>