diff -r 19efc2af3e6c -r f967a16dfcdd src/HOL/Nitpick_Examples/Manual_Nits.thy --- a/src/HOL/Nitpick_Examples/Manual_Nits.thy Mon Sep 06 22:58:06 2010 +0200 +++ b/src/HOL/Nitpick_Examples/Manual_Nits.thy Tue Sep 07 10:05:19 2010 +0200 @@ -110,7 +110,7 @@ "my_int_rel (x, y) (u, v) = (x + v = u + y)" quotient_type my_int = "nat \ nat" / my_int_rel -by (auto simp add: equivp_def expand_fun_eq) +by (auto simp add: equivp_def ext_iff) definition add_raw where "add_raw \ \(x, y) (u, v). (x + (u\nat), y + (v\nat))"