src/HOL/Predicate_Compile_Examples/Hotel_Example.thy
changeset 39200 bb93713b0925
parent 39189 d183bf90dabd
parent 39198 f967a16dfcdd
child 39302 d7728f65b353
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Tue Sep 07 11:52:43 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Tue Sep 07 12:04:34 2010 +0200
@@ -79,10 +79,10 @@
 declare Let_def[code_pred_inline]
 
 lemma [code_pred_inline]: "insert == (%y A x. y = x | A x)"
-by (auto simp add: insert_iff[unfolded mem_def] expand_fun_eq intro!: eq_reflection)
+by (auto simp add: insert_iff[unfolded mem_def] ext_iff intro!: eq_reflection)
 
 lemma [code_pred_inline]: "(op -) == (%A B x. A x \<and> \<not> B x)"
-by (auto simp add: Diff_iff[unfolded mem_def] expand_fun_eq intro!: eq_reflection)
+by (auto simp add: Diff_iff[unfolded mem_def] ext_iff intro!: eq_reflection)
 
 setup {* Code_Prolog.map_code_options (K
   {ensure_groundness = true,