src/HOL/Datatype_Universe.thy
changeset 11451 8abfb4f7bd02
parent 10832 e33b47e4246d
child 11483 f4d10044a2cd
--- a/src/HOL/Datatype_Universe.thy	Tue Jul 24 11:25:54 2001 +0200
+++ b/src/HOL/Datatype_Universe.thy	Wed Jul 25 13:13:01 2001 +0200
@@ -9,7 +9,7 @@
 Could <*> be generalized to a general summation (Sigma)?
 *)
 
-Datatype_Universe = NatArith + Sum_Type +
+Datatype_Universe = NatArith + Sum_Type + Hilbert_Choice +
 
 
 (** lists, trees will be sets of nodes **)
@@ -86,10 +86,10 @@
   usum_def   "usum A B == In0`A Un In1`B"
 
   (*the corresponding eliminators*)
-  Split_def  "Split c M == @u. ? x y. M = Scons x y & u = c x y"
+  Split_def  "Split c M == THE u. EX x y. M = Scons x y & u = c x y"
 
-  Case_def   "Case c d M == @u.  (? x . M = In0(x) & u = c(x)) 
-                               | (? y . M = In1(y) & u = d(y))"
+  Case_def   "Case c d M == THE u.  (EX x . M = In0(x) & u = c(x)) 
+                                  | (EX y . M = In1(y) & u = d(y))"
 
 
   (** equality for the "universe" **)