src/HOL/AxClasses/Group/Group.thy
author paulson
Thu, 08 Jan 1998 11:23:18 +0100
changeset 4522 0218c486cf07
parent 2907 0e272e4c7cb2
permissions -rw-r--r--
Restored the ciphertext in OR4 in order to make the spec closer to that in OtwayRees.thy

(*  Title:      Group.thy
    ID:         $Id$
    Author:     Markus Wenzel, TU Muenchen
*)

Group = Sigs + Fun +

(* semigroups *)

axclass
  semigroup < times
  assoc         "(x * y) * z = x * (y * z)"


(* groups *)

axclass
  group < one, inverse, semigroup
  left_unit     "1 * x = x"
  left_inverse  "inverse x * x = 1"


(* abelian groups *)

axclass
  agroup < group
  commut        "x * y = y * x"

end