diff -r 38e5c05ef741 -r 5a3e336a2e37 src/HOL/Complex/ex/ReflectedFerrack.thy --- a/src/HOL/Complex/ex/ReflectedFerrack.thy Sun Sep 30 16:53:08 2007 +0200 +++ b/src/HOL/Complex/ex/ReflectedFerrack.thy Sun Sep 30 21:55:15 2007 +0200 @@ -1908,7 +1908,7 @@ from alluopairs_set1[where xs="?U"] have UpU: "set ?Up \ (set ?U \ set ?U)" by simp from uset_l[OF lq] have U_l: "\ (t,n) \ set ?U. numbound0 t \ n > 0" . from U_l UpU - have Up_: "\ ((t,n),(s,m)) \ set ?Up. numbound0 t \ n> 0 \ numbound0 s \ m > 0" by auto + have "\ ((t,n),(s,m)) \ set ?Up. numbound0 t \ n> 0 \ numbound0 s \ m > 0" by auto hence Snb: "\ (t,n) \ set ?S. numbound0 t \ n > 0 " by (auto simp add: mult_pos_pos) have Y_l: "\ (t,n) \ set ?Y. numbound0 t \ n > 0"