doc-src/TutorialI/Types/Overloading.thy
changeset 38325 6daf896bca5e
parent 36176 3fe7e97ccca8
--- a/doc-src/TutorialI/Types/Overloading.thy	Wed Aug 11 12:03:57 2010 +0200
+++ b/doc-src/TutorialI/Types/Overloading.thy	Wed Aug 11 12:04:06 2010 +0200
@@ -55,10 +55,10 @@
 text {* \noindent From now on, terms like @{term "Suc (m \<oplus> 2)"} are
 legal. *}
 
-instantiation "*" :: (plus, plus) plus
+instantiation prod :: (plus, plus) plus
 begin
 
-text {* \noindent Here we instantiate the product type @{type "*"} to
+text {* \noindent Here we instantiate the product type @{type prod} to
 class @{class [source] plus}, given that its type arguments are of
 class @{class [source] plus}: *}