src/HOL/Prod.thy
changeset 2886 fd5645efa43d
parent 2880 a0fde30aa126
child 2973 184c7cd8043d
--- a/src/HOL/Prod.thy	Thu Apr 03 10:36:54 1997 +0200
+++ b/src/HOL/Prod.thy	Thu Apr 03 19:29:53 1997 +0200
@@ -79,7 +79,7 @@
 
 (** unit **)
 
-typedef  unit = "{p. p = True}"
+typedef  unit = "{True}"
 
 consts
   "()"          :: unit                           ("'(')")