doc-src/AxClass/Group/Product.thy
changeset 9146 dde1affac73e
parent 8907 813fabceec00
child 9306 d0ef4a41ae63
--- a/doc-src/AxClass/Group/Product.thy	Mon Jun 26 11:21:49 2000 +0200
+++ b/doc-src/AxClass/Group/Product.thy	Mon Jun 26 11:43:56 2000 +0200
@@ -1,7 +1,7 @@
 
-header {* Syntactic classes *};
+header {* Syntactic classes *}
 
-theory Product = Main:;
+theory Product = Main:
 
 text {*
  \medskip\noindent There is still a feature of Isabelle's type system
@@ -16,12 +16,12 @@
 
  The $product$ class below provides a less degenerate example of
  syntactic type classes.
-*};
+*}
 
 axclass
-  product < "term";
+  product < "term"
 consts
-  product :: "'a::product \\<Rightarrow> 'a \\<Rightarrow> 'a"    (infixl "\\<Otimes>" 70);
+  product :: "'a::product \\<Rightarrow> 'a \\<Rightarrow> 'a"    (infixl "\\<Otimes>" 70)
 
 text {*
  Here class $product$ is defined as subclass of $term$ without any
@@ -50,12 +50,12 @@
  certain type $\tau$ do we instantiate $\tau :: c$.
 
  This is done for class $product$ and type $bool$ as follows.
-*};
+*}
 
-instance bool :: product;
-  by intro_classes;
+instance bool :: product
+  by intro_classes
 defs
-  product_bool_def: "x \\<Otimes> y \\<equiv> x \\<and> y";
+  product_bool_def: "x \\<Otimes> y \\<equiv> x \\<and> y"
 
 text {*
  The definition $prod_bool_def$ becomes syntactically well-formed only
@@ -78,6 +78,6 @@
  This style of \texttt{instance} won't make much sense in Isabelle's
  meta-logic, because there is no internal notion of ``providing
  operations'' or even ``names of functions''.
-*};
+*}
 
-end;
\ No newline at end of file
+end
\ No newline at end of file