doc-src/TutorialI/Types/Overloading1.thy
changeset 12338 de0f4a63baa5
parent 11494 23a118849801
child 12815 1f073030b97a
--- a/doc-src/TutorialI/Types/Overloading1.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/doc-src/TutorialI/Types/Overloading1.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -10,13 +10,12 @@
 introduce the class @{text ordrel}:
 *}
 
-axclass ordrel < "term"
+axclass ordrel < type
 
 text{*\noindent
 This introduces a new class @{text ordrel} and makes it a subclass of
-the predefined class @{text term}, which
-is the class of all HOL types.\footnote{The quotes around @{text term}
-simply avoid the clash with the command \isacommand{term}.}
+the predefined class @{text type}, which
+is the class of all HOL types.
 This is a degenerate form of axiomatic type class without any axioms.
 Its sole purpose is to restrict the use of overloaded constants to meaningful
 instances: