src/HOL/Algebra/Group.thy
changeset 14551 2cb6ff394bfb
parent 14286 0ae66ffb9784
child 14651 02b8f3bcf7fe
--- a/src/HOL/Algebra/Group.thy	Tue Apr 13 07:48:32 2004 +0200
+++ b/src/HOL/Algebra/Group.thy	Tue Apr 13 09:42:40 2004 +0200
@@ -410,6 +410,7 @@
   shows "semigroup (G(| carrier := H |))"
   using prems by fast
 
+
 locale subgroup = submagma H G +
   assumes one_closed [intro, simp]: "\<one> \<in> H"
     and m_inv_closed [intro, simp]: "x \<in> H ==> inv x \<in> H"