src/HOL/Predicate_Compile.thy
changeset 69593 3dda49e08b9d
parent 67613 ce654b0e6d69
child 69605 a96320074298
--- a/src/HOL/Predicate_Compile.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Predicate_Compile.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -80,14 +80,14 @@
   val ii = Fun (Input, Fun (Input, Bool))
 in
   Core_Data.PredData.map (Graph.new_node 
-    (@{const_name contains}, 
+    (\<^const_name>\<open>contains\<close>, 
      Core_Data.PredData {
        pos = Position.thread_data (),
        intros = [(NONE, @{thm containsI})], 
        elim = SOME @{thm containsE}, 
        preprocessed = true,
        function_names = [(Predicate_Compile_Aux.Pred, 
-         [(io, @{const_name pred_of_set}), (ii, @{const_name contains_pred})])], 
+         [(io, \<^const_name>\<open>pred_of_set\<close>), (ii, \<^const_name>\<open>contains_pred\<close>)])], 
        predfun_data = [
          (io, Core_Data.PredfunData {
             elim = @{thm pred_of_setE}, intro = @{thm pred_of_setI},