src/HOL/Library/datatype_records.ML
changeset 69593 3dda49e08b9d
parent 68910 a21202dfe3eb
child 69598 81caae4fc4fa
--- a/src/HOL/Library/datatype_records.ML	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Library/datatype_records.ML	Fri Jan 04 23:22:53 2019 +0100
@@ -36,7 +36,7 @@
 )
 
 fun mk_eq_dummy (lhs, rhs) =
-  Const (@{const_name HOL.eq}, dummyT --> dummyT --> @{typ bool}) $ lhs $ rhs
+  Const (\<^const_name>\<open>HOL.eq\<close>, dummyT --> dummyT --> \<^typ>\<open>bool\<close>) $ lhs $ rhs
 
 val dummify = map_types (K dummyT)
 fun repeat_split_tac ctxt thm = REPEAT_ALL_NEW (CHANGED o Splitter.split_tac ctxt [thm])
@@ -278,7 +278,7 @@
           NONE => raise Fail ("not a valid record field: " ^ name)
         | SOME s => Const (s, dummyT) $ Abs (Name.uu_, dummyT, arg)
       end
-  | field_update_tr _ t = raise TERM ("field_update_tr", [@{print} t]);
+  | field_update_tr _ t = raise TERM ("field_update_tr", [\<^print> t]);
 
 fun field_updates_tr ctxt (Const (\<^syntax_const>\<open>_datatype_field_updates\<close>, _) $ t $ u) =
       field_update_tr ctxt t :: field_updates_tr ctxt u
@@ -291,7 +291,7 @@
   | record_update_tr _ ts = raise TERM ("record_update_tr", ts);
 
 val parse_ctr_options =
-  Scan.optional (@{keyword "("} |-- Parse.list1 (Plugin_Name.parse_filter >> K) --| @{keyword ")"} >>
+  Scan.optional (\<^keyword>\<open>(\<close> |-- Parse.list1 (Plugin_Name.parse_filter >> K) --| \<^keyword>\<open>)\<close> >>
     (fn fs => fold I fs default_ctr_options_cmd)) default_ctr_options_cmd
 
 val parser =
@@ -300,7 +300,7 @@
 
 val _ =
   Outer_Syntax.local_theory
-    @{command_keyword datatype_record}
+    \<^command_keyword>\<open>datatype_record\<close>
     "Defines a record based on the BNF/datatype machinery"
     (parser >> (fn (((ctr_options, tyargs), binding), args) =>
       record_cmd binding ctr_options tyargs args))