src/HOL/AxClasses/Semigroups.thy
changeset 30152 0ddd8028f98c
parent 30151 629f3a92863e
parent 30148 5d04b67a866e
child 30153 051d3825a15d
--- a/src/HOL/AxClasses/Semigroups.thy	Thu Feb 26 10:13:43 2009 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,21 +0,0 @@
-(*  Title:      HOL/AxClasses/Semigroups.thy
-    ID:         $Id$
-    Author:     Markus Wenzel, TU Muenchen
-*)
-
-theory Semigroups imports Main begin
-
-consts
-  times :: "'a => 'a => 'a"    (infixl "[*]" 70)
-
-axclass semigroup < type
-  assoc: "(x [*] y) [*] z = x [*] (y [*] z)"
-
-
-consts
-  plus :: "'a => 'a => 'a"    (infixl "[+]" 70)
-
-axclass plus_semigroup < type
-  assoc: "(x [+] y) [+] z = x [+] (y [+] z)"
-
-end