doc-src/TutorialI/Types/Overloading0.thy
changeset 12332 aea72a834c85
parent 11494 23a118849801
child 17914 99ead7a7eb42
--- a/doc-src/TutorialI/Types/Overloading0.thy	Thu Nov 29 20:02:23 2001 +0100
+++ b/doc-src/TutorialI/Types/Overloading0.thy	Thu Nov 29 21:12:37 2001 +0100
@@ -35,7 +35,7 @@
 However, there is nothing to prevent the user from forming terms such as
 @{text"inverse []"} and proving theorems such as @{text"inverse []
 = inverse []"} when inverse is not defined on lists.  Proving theorems about
-undefined constants does not endanger soundness, but it is pointless.
+unspecified constants does not endanger soundness, but it is pointless.
 To prevent such terms from even being formed requires the use of type classes.
 *}
 (*<*)end(*>*)