HOL.thy
changeset 41 054ce38225b9
parent 38 7ef6ba42914b
child 49 9f35f2744fa8
--- a/HOL.thy	Thu Feb 03 09:55:47 1994 +0100
+++ b/HOL.thy	Fri Feb 11 11:09:50 1994 +0100
@@ -103,7 +103,7 @@
 
   (* Definitions *)
 
-  True_def      "True = ((%x.x)=(%x.x))"
+  True_def      "True = ((%x::bool.x)=(%x.x))"
   All_def       "All  = (%P. P = (%x.True))"
   Ex_def        "Ex   = (%P. P(@x.P(x)))"
   False_def     "False = (!P.P)"