src/HOL/Library/Function_Algebras.thy
changeset 39302 d7728f65b353
parent 39198 f967a16dfcdd
child 46575 f1e387195a56
--- a/src/HOL/Library/Function_Algebras.thy	Mon Sep 13 08:43:48 2010 +0200
+++ b/src/HOL/Library/Function_Algebras.thy	Mon Sep 13 11:13:15 2010 +0200
@@ -57,7 +57,7 @@
 qed (simp add: plus_fun_def add.assoc)
 
 instance "fun" :: (type, cancel_semigroup_add) cancel_semigroup_add proof
-qed (simp_all add: plus_fun_def ext_iff)
+qed (simp_all add: plus_fun_def fun_eq_iff)
 
 instance "fun" :: (type, ab_semigroup_add) ab_semigroup_add proof
 qed (simp add: plus_fun_def add.commute)
@@ -106,7 +106,7 @@
 qed (simp_all add: zero_fun_def times_fun_def)
 
 instance "fun" :: (type, zero_neq_one) zero_neq_one proof
-qed (simp add: zero_fun_def one_fun_def ext_iff)
+qed (simp add: zero_fun_def one_fun_def fun_eq_iff)
 
 
 text {* Ring structures *}