spurious set/pred correction
authorhaftmann
Sat, 03 Mar 2012 21:00:31 +0100
changeset 46782 d50855d9ea74
parent 46781 4ec6bd791ee9
child 46783 3e89a5cab8d7
spurious set/pred correction
src/HOL/Import/HOLLightCompat.thy
--- a/src/HOL/Import/HOLLightCompat.thy	Sat Mar 03 21:00:24 2012 +0100
+++ b/src/HOL/Import/HOLLightCompat.thy	Sat Mar 03 21:00:31 2012 +0100
@@ -192,8 +192,8 @@
   by auto
 
 lemma DEF_INSERT:
-  "insert = (%u ua y. y \<in> ua | y = u)"
-  unfolding mem_def fun_eq_iff insert_code by blast
+  "insert = (\<lambda>u ua. {y. y \<in> ua | y = u})"
+  by auto
 
 lemma DEF_IMAGE:
   "op ` = (\<lambda>u ua. {ub. \<exists>y. (\<exists>x. x \<in> ua \<and> y = u x) \<and> ub = y})"
@@ -331,8 +331,8 @@
 
 lemmas [hol4rew] = id_apply
 
-lemma DEF_CHOICE: "Eps = (%u. SOME x. x \<in> u)"
-  by (simp add: mem_def)
+lemma DEF_CHOICE: "Eps = (%u. SOME x. u x)"
+  by simp
 
 definition dotdot :: "nat => nat => nat set"
   where "dotdot u ua = {ub. EX x. (u <= x & x <= ua) & ub = x}"
@@ -347,3 +347,4 @@
   by (simp add: INFINITE_def_raw)
 
 end
+