diff -r e1bd8a54c40f -r d7728f65b353 src/HOL/Library/Enum.thy --- a/src/HOL/Library/Enum.thy Mon Sep 13 08:43:48 2010 +0200 +++ b/src/HOL/Library/Enum.thy Mon Sep 13 11:13:15 2010 +0200 @@ -42,7 +42,7 @@ "HOL.equal f g \ (\x \ set enum. f x = g x)" instance proof -qed (simp_all add: equal_fun_def enum_all ext_iff) +qed (simp_all add: equal_fun_def enum_all fun_eq_iff) end @@ -54,7 +54,7 @@ fixes f g :: "'a\enum \ 'b\order" shows "f \ g \ list_all (\x. f x \ g x) enum" and "f < g \ f \ g \ list_ex (\x. f x \ g x) enum" - by (simp_all add: list_all_iff list_ex_iff enum_all ext_iff le_fun_def order_less_le) + by (simp_all add: list_all_iff list_ex_iff enum_all fun_eq_iff le_fun_def order_less_le) subsection {* Quantifiers *} @@ -82,7 +82,7 @@ by (induct n arbitrary: ys) auto lemma set_n_lists: "set (n_lists n xs) = {ys. length ys = n \ set ys \ set xs}" -proof (rule set_ext) +proof (rule set_eqI) fix ys :: "'a list" show "ys \ set (n_lists n xs) \ ys \ {ys. length ys = n \ set ys \ set xs}" proof - @@ -160,7 +160,7 @@ proof (rule UNIV_eq_I) fix f :: "'a \ 'b" have "f = the \ map_of (zip (enum \ 'a\enum list) (map f enum))" - by (auto simp add: map_of_zip_map ext_iff) + by (auto simp add: map_of_zip_map fun_eq_iff) then show "f \ set enum" by (auto simp add: enum_fun_def set_n_lists) qed