src/HOL/Algebra/Divisibility.thy
changeset 75455 91c16c5ad3e9
parent 73706 4b1386b2c23e
child 80914 d97fdabd9e2b
--- a/src/HOL/Algebra/Divisibility.thy	Wed May 11 10:42:24 2022 +0200
+++ b/src/HOL/Algebra/Divisibility.thy	Tue May 17 14:10:14 2022 +0100
@@ -2600,7 +2600,7 @@
 next
   case (Cons x as)
   then have "x \<in> carrier G"  "set as \<subseteq> carrier G" and "a divides x \<otimes> foldr (\<otimes>) as \<one>"
-    by (auto simp: )
+    by auto
   with carr aprime have "a divides x \<or> a divides foldr (\<otimes>) as \<one>"
     by (intro prime_divides) simp+
   then show ?case