src/HOL/Algebra/Ideal.thy
changeset 27698 197f0517f0bd
parent 27611 2c01c0bdb385
child 27714 27b4d7c01f8b
--- a/src/HOL/Algebra/Ideal.thy	Tue Jul 29 16:16:10 2008 +0200
+++ b/src/HOL/Algebra/Ideal.thy	Tue Jul 29 16:17:13 2008 +0200
@@ -950,7 +950,7 @@
         have aUnit: "a \<in> Units R" by (simp add: field_Units)
     hence a: "a \<otimes> inv a = \<one>" by (rule Units_r_inv)
     from aI and aUnit
-        have "a \<otimes> inv a \<in> I" by (simp add: I_r_closed)
+        have "a \<otimes> inv a \<in> I" by (simp add: I_r_closed del: Units_r_inv)
     hence oneI: "\<one> \<in> I" by (simp add: a[symmetric])
 
     have "carrier R \<subseteq> I"