src/HOL/AxClasses/Tutorial/Product.thy
author wenzelm
Mon, 22 May 2000 16:04:32 +0200
changeset 8922 490637ba1d7f
parent 8920 af5e09b6c208
child 9363 86b48eafc70d
permissions -rw-r--r--
tuned;

(*  Title:      HOL/AxClasses/Tutorial/Product.thy
    ID:         $Id$
    Author:     Markus Wenzel, TU Muenchen
*)

theory Product = Main:;

axclass
  product < "term";
consts
  product :: "'a::product => 'a => 'a"    (infixl "[*]" 70);

instance bool :: product;
  by intro_classes;
defs
  product_bool_def: "x [*] y == x & y";

end;