src/HOL/Bali/State.thy
changeset 14766 c0401da7726d
parent 14171 0cab06e3bbd0
child 14981 e73f8140af78
--- a/src/HOL/Bali/State.thy	Fri May 21 21:14:18 2004 +0200
+++ b/src/HOL/Bali/State.thy	Fri May 21 21:14:52 2004 +0200
@@ -41,7 +41,7 @@
 constdefs
   
   the_Arr :: "obj option \<Rightarrow> ty \<times> int \<times> (vn, val) table"
- "the_Arr obj \<equiv> \<epsilon>(T,k,t). obj = Some \<lparr>tag=Arr T k,values=t\<rparr>"
+ "the_Arr obj \<equiv> SOME (T,k,t). obj = Some \<lparr>tag=Arr T k,values=t\<rparr>"
 
 lemma the_Arr_Arr [simp]: "the_Arr (Some \<lparr>tag=Arr T k,values=cs\<rparr>) = (T,k,cs)"
 apply (auto simp: the_Arr_def)
@@ -266,7 +266,7 @@
 
 constdefs
   new_Addr     :: "heap \<Rightarrow> loc option"
- "new_Addr h   \<equiv> if (\<forall>a. h a \<noteq> None) then None else Some (\<epsilon> a. h a = None)"
+ "new_Addr h   \<equiv> if (\<forall>a. h a \<noteq> None) then None else Some (SOME a. h a = None)"
 
 lemma new_AddrD: "new_Addr h = Some a \<Longrightarrow> h a = None"
 apply (unfold new_Addr_def)