src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy
changeset 67399 eab6ce8368fa
parent 66453 cc19f7ca2ed6
child 67613 ce654b0e6d69
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example_Prolog.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -11,7 +11,7 @@
 lemma [code_pred_inline]: "insert == (%y A x. y = x | A x)"
 by (auto simp add: insert_iff[unfolded mem_def] fun_eq_iff intro!: eq_reflection)
 
-lemma [code_pred_inline]: "(op -) == (%A B x. A x \<and> \<not> B x)"
+lemma [code_pred_inline]: "(-) == (%A B x. A x \<and> \<not> B x)"
 by (auto simp add: Diff_iff[unfolded mem_def] fun_eq_iff intro!: eq_reflection)
 *)