src/HOL/Tools/BNF/bnf_lfp_rec_sugar.ML
changeset 69593 3dda49e08b9d
parent 67522 9e712280cc37
child 69992 bd3c10813cc4
--- a/src/HOL/Tools/BNF/bnf_lfp_rec_sugar.ML	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Tools/BNF/bnf_lfp_rec_sugar.ML	Fri Jan 04 23:22:53 2019 +0100
@@ -274,7 +274,7 @@
       induct_attrs, map #T basic_lfp_sugars), lthy)
   end;
 
-val undef_const = Const (@{const_name undefined}, dummyT);
+val undef_const = Const (\<^const_name>\<open>undefined\<close>, dummyT);
 
 type eqn_data = {
   fun_name: string,
@@ -677,10 +677,10 @@
    || Parse.reserved "nonexhaustive" >> K Nonexhaustive_Option
    || Parse.reserved "transfer" >> K Transfer_Option);
 
-val _ = Outer_Syntax.local_theory @{command_keyword primrec}
+val _ = Outer_Syntax.local_theory \<^command_keyword>\<open>primrec\<close>
   "define primitive recursive functions"
-  ((Scan.optional (@{keyword "("} |-- Parse.!!! (Parse.list1 rec_option_parser)
-      --| @{keyword ")"}) []) -- Parse_Spec.specification
+  ((Scan.optional (\<^keyword>\<open>(\<close> |-- Parse.!!! (Parse.list1 rec_option_parser)
+      --| \<^keyword>\<open>)\<close>) []) -- Parse_Spec.specification
     >> (fn (opts, (fixes, specs)) => snd o primrec_cmd true opts fixes specs));
 
 end;