src/HOL/Quotient_Examples/Quotient_Int.thy
changeset 39302 d7728f65b353
parent 39198 f967a16dfcdd
child 40468 d4aac200199e
--- a/src/HOL/Quotient_Examples/Quotient_Int.thy	Mon Sep 13 08:43:48 2010 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_Int.thy	Mon Sep 13 11:13:15 2010 +0200
@@ -14,7 +14,7 @@
   "intrel (x, y) (u, v) = (x + v = u + y)"
 
 quotient_type int = "nat \<times> nat" / intrel
-  by (auto simp add: equivp_def ext_iff)
+  by (auto simp add: equivp_def fun_eq_iff)
 
 instantiation int :: "{zero, one, plus, uminus, minus, times, ord, abs, sgn}"
 begin