src/HOL/Algebra/Coset.thy
changeset 16417 9bc16273c2d4
parent 15120 f0359f75682e
child 19380 b808efaa5828
--- a/src/HOL/Algebra/Coset.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Algebra/Coset.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 
 header{*Cosets and Quotient Groups*}
 
-theory Coset = Group + Exponent:
+theory Coset imports Group Exponent begin
 
 constdefs (structure G)
   r_coset    :: "[_, 'a set, 'a] \<Rightarrow> 'a set"    (infixl "#>\<index>" 60)