src/HOL/AxClasses/Group/Monoid.thy
author clasohm
Wed, 20 Mar 1996 13:21:12 +0100
changeset 1589 fd6a571cb2b0
parent 1247 18b1441fb603
permissions -rw-r--r--
added warning and automatic deactivation of HTML generation if we cannot write .theory_list.txt; fixed bug which occured when index_path's value is "/"
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1247
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     1
(*  Title:      Monoid.thy
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     3
    Author:     Markus Wenzel, TU Muenchen
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     4
*)
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     5
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     6
Monoid = Sigs +
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     7
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     8
(* monoids *)
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
     9
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    10
axclass
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    11
  monoid < times, one
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    12
  assoc         "(x * y) * z = x * (y * z)"
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    13
  left_unit     "1 * x = x"
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    14
  right_unit    "x * 1 = x"
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    15
18b1441fb603 Various axiomatic type class demos;
wenzelm
parents:
diff changeset
    16
end