put expand_(fun/set)_eq back in as synonyms, for compatibility
authornipkow
Wed, 08 Sep 2010 10:45:55 +0200
changeset 39213 297cd703f1f0
parent 39212 3989b2b44dba
child 39214 49fc6c842d6c
child 39216 62332b382dba
put expand_(fun/set)_eq back in as synonyms, for compatibility
src/HOL/Fun.thy
src/HOL/Set.thy
--- a/src/HOL/Fun.thy	Tue Sep 07 15:56:33 2010 -0700
+++ b/src/HOL/Fun.thy	Wed Sep 08 10:45:55 2010 +0200
@@ -18,6 +18,8 @@
 apply (simp (no_asm_simp))
 done
 
+lemmas expand_fun_eq = ext_iff
+
 lemma apply_inverse:
   "f x = u \<Longrightarrow> (\<And>x. P x \<Longrightarrow> g (f x) = x) \<Longrightarrow> P x \<Longrightarrow> x = g u"
   by auto
--- a/src/HOL/Set.thy	Tue Sep 07 15:56:33 2010 -0700
+++ b/src/HOL/Set.thy	Wed Sep 08 10:45:55 2010 +0200
@@ -498,6 +498,8 @@
 lemma set_ext_iff [no_atp]: "(A = B) = (ALL x. (x:A) = (x:B))"
 by(auto intro:set_ext)
 
+lemmas expand_set_eq [no_atp] = set_ext_iff
+
 lemma subset_antisym [intro!]: "A \<subseteq> B ==> B \<subseteq> A ==> A = B"
   -- {* Anti-symmetry of the subset relation. *}
   by (iprover intro: set_ext subsetD)