doc-src/AxClass/Group/Semigroup.thy
changeset 8906 fc7841f31388
parent 8905 4f0f79fe41b9
child 8907 813fabceec00
equal deleted inserted replaced
8905:4f0f79fe41b9 8906:fc7841f31388
     1 theory Semigroup = Main:;
       
     2 
       
     3 consts
       
     4   times :: "'a \\<Rightarrow> 'a \\<Rightarrow> 'a"    (infixl "\<Otimes>" 70);
       
     5 axclass
       
     6   semigroup < "term"
       
     7   assoc: "(x \<Otimes> y) \<Otimes> z = x \<Otimes> (y \<Otimes> z)";
       
     8 
       
     9 end;