src/HOL/Product_Type.thy
changeset 11602 bf6700f4c010
parent 11493 f3ff2549cdc8
child 11777 b03c8a3fcc6d
--- a/src/HOL/Product_Type.thy	Thu Sep 27 22:22:08 2001 +0200
+++ b/src/HOL/Product_Type.thy	Thu Sep 27 22:22:58 2001 +0200
@@ -96,21 +96,15 @@
 
 (** unit **)
 
-global
-
 typedef unit = "{True}"
 proof
   show "True : ?unit"
     by blast
 qed
 
-consts
-  "()"          :: unit                           ("'(')")
-
-local
-
-defs
-  Unity_def:    "() == Abs_unit True"
+constdefs
+  Unity :: unit    ("'(')")
+  "() == Abs_unit True"