src/HOL/Bali/State.thy
changeset 18576 8d98b7711e47
parent 18447 da548623916a
child 25511 54db9b5080b8
--- a/src/HOL/Bali/State.thy	Wed Jan 04 17:04:11 2006 +0100
+++ b/src/HOL/Bali/State.thy	Wed Jan 04 19:22:53 2006 +0100
@@ -268,7 +268,7 @@
  "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 (auto simp add: not_Some_eq new_Addr_def)
+apply (auto simp add: new_Addr_def)
 apply (erule someI) 
 done
 
@@ -278,7 +278,7 @@
 done
 
 lemma new_Addr_SomeI: "h a = None \<Longrightarrow> \<exists>b. new_Addr h = Some b \<and> h b = None"
-apply (simp add: new_Addr_def not_Some_eq)
+apply (simp add: new_Addr_def)
 apply (fast intro: someI2)
 done