src/HOL/ex/Commands.thy
changeset 69597 ff784d5a5bfb
parent 67096 e77f13a6a501
child 70308 7f568724d67e
--- a/src/HOL/ex/Commands.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/ex/Commands.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -15,7 +15,7 @@
 subsection \<open>Diagnostic command: no state change\<close>
 
 ML \<open>
-  Outer_Syntax.command @{command_keyword print_test} "print term test"
+  Outer_Syntax.command \<^command_keyword>\<open>print_test\<close> "print term test"
     (Parse.term >> (fn s => Toplevel.keep (fn st =>
       let
         val ctxt = Toplevel.context_of st;
@@ -31,10 +31,10 @@
 subsection \<open>Old-style global theory declaration\<close>
 
 ML \<open>
-  Outer_Syntax.command @{command_keyword global_test} "test constant declaration"
+  Outer_Syntax.command \<^command_keyword>\<open>global_test\<close> "test constant declaration"
     (Parse.binding >> (fn b => Toplevel.theory (fn thy =>
       let
-        val thy' = Sign.add_consts [(b, @{typ 'a}, NoSyn)] thy;
+        val thy' = Sign.add_consts [(b, \<^typ>\<open>'a\<close>, NoSyn)] thy;
       in thy' end)));
 \<close>
 
@@ -46,8 +46,8 @@
 subsection \<open>Local theory specification\<close>
 
 ML \<open>
-  Outer_Syntax.local_theory @{command_keyword local_test} "test local definition"
-    (Parse.binding -- (@{keyword "="} |-- Parse.term) >> (fn (b, s) => fn lthy =>
+  Outer_Syntax.local_theory \<^command_keyword>\<open>local_test\<close> "test local definition"
+    (Parse.binding -- (\<^keyword>\<open>=\<close> |-- Parse.term) >> (fn (b, s) => fn lthy =>
       let
         val t = Syntax.read_term lthy s;
         val (def, lthy') = Local_Theory.define ((b, NoSyn), ((Thm.def_binding b, []), t)) lthy;