src/HOL/Algebra/Divisibility.thy
changeset 68399 0b71d08528f0
parent 68004 a8a20be7053a
child 68470 7ddcce75c3ee
--- a/src/HOL/Algebra/Divisibility.thy	Tue Jun 05 16:35:52 2018 +0200
+++ b/src/HOL/Algebra/Divisibility.thy	Wed Jun 06 14:25:53 2018 +0100
@@ -50,14 +50,6 @@
 
 subsection \<open>Products of Units in Monoids\<close>
 
-lemma (in monoid) Units_m_closed[simp, intro]:
-  assumes h1unit: "h1 \<in> Units G"
-    and h2unit: "h2 \<in> Units G"
-  shows "h1 \<otimes> h2 \<in> Units G"
-  unfolding Units_def
-  using assms
-  by auto (metis Units_inv_closed Units_l_inv Units_m_closed Units_r_inv)
-
 lemma (in monoid) prod_unit_l:
   assumes abunit[simp]: "a \<otimes> b \<in> Units G"
     and aunit[simp]: "a \<in> Units G"