doc-src/AxClass/Group/Semigroup.thy
author wenzelm
Sun, 21 May 2000 01:12:00 +0200
changeset 8890 9a44d8d98731
permissions -rw-r--r--
snapshot of new Isar'ized version;

theory Semigroup = Main:;

consts
  times :: "'a \\<Rightarrow> 'a \\<Rightarrow> 'a"    (infixl "\<Otimes>" 70);
axclass
  semigroup < "term"
  assoc: "(x \<Otimes> y) \<Otimes> z = x \<Otimes> (y \<Otimes> z)";

end;