src/HOL/AxClasses/Product.thy
changeset 12338 de0f4a63baa5
parent 10681 ec76e17f73c5
child 14981 e73f8140af78
--- a/src/HOL/AxClasses/Product.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/src/HOL/AxClasses/Product.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -6,7 +6,7 @@
 
 theory Product = Main:
 
-axclass product < "term"
+axclass product < type
 
 consts
   product :: "'a::product => 'a => 'a"    (infixl "[*]" 70)