src/HOL/AxClasses/Group/GroupDefs.thy
author paulson
Tue, 16 Jul 1996 15:49:46 +0200
changeset 1868 836950047d85
parent 1247 18b1441fb603
child 2907 0e272e4c7cb2
permissions -rw-r--r--
Put in minimal simpset to avoid excessive simplification, just as in revision 1.9 of HOL/indrule.ML

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

GroupDefs = MonoidGroupInsts + Prod + Fun +


(* bool *)

instance
  bool :: {times, inv, one}

defs
  times_bool_def        "x * y == (x ~= y)"
  inv_bool_def          "inv x == (x::bool)"
  one_bool_def          "1 == False"


(* cartesian products *)

instance
  "*" :: (term, term) {times, inv, one}

defs
  times_prod_def        "p * q == (fst p * fst q, snd p * snd q)"
  inv_prod_def          "inv p == (inv (fst p), inv (snd p))"
  one_prod_def          "1 == (1, 1)"


(* function spaces *)

instance
  fun :: (term, term) {times, inv, one}

defs
  times_fun_def         "f * g == (%x. f x * g x)"
  inv_fun_def           "inv f == (%x. inv (f x))"
  one_fun_def           "1 == (%x. 1)"

end