src/HOL/ex/Classpackage.thy
changeset 22424 8a5412121687
parent 22384 33a46e6c7f04
child 22473 753123c89d72
--- a/src/HOL/ex/Classpackage.thy	Fri Mar 09 08:45:53 2007 +0100
+++ b/src/HOL/ex/Classpackage.thy	Fri Mar 09 08:45:55 2007 +0100
@@ -2,7 +2,7 @@
     Author:     Florian Haftmann, TU Muenchen
 *)
 
-header {* Test and examples for new class package *}
+header {* Test and examples for Isar class package *}
 
 theory Classpackage
 imports Main
@@ -328,6 +328,7 @@
 instance * :: (group_comm, group_comm) group_comm
 by default (simp_all add: split_paired_all mult_prod_def comm)
 
+ 
 definition
   "X a b c = (a \<otimes> \<one> \<otimes> b, a \<otimes> \<one> \<otimes> b, [a, b] \<otimes> \<one> \<otimes> [a, b, c])"
 definition