src/HOL/AxClasses/Semigroups.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
--- a/src/HOL/AxClasses/Semigroups.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/AxClasses/Semigroups.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -3,7 +3,7 @@
     Author:     Markus Wenzel, TU Muenchen
 *)
 
-theory Semigroups = Main:
+theory Semigroups imports Main begin
 
 consts
   times :: "'a => 'a => 'a"    (infixl "[*]" 70)