src/HOL/Unix/Unix.thy
changeset 18576 8d98b7711e47
parent 18447 da548623916a
child 18730 843da46f89ac
--- a/src/HOL/Unix/Unix.thy	Wed Jan 04 17:04:11 2006 +0100
+++ b/src/HOL/Unix/Unix.thy	Wed Jan 04 19:22:53 2006 +0100
@@ -1059,7 +1059,7 @@
                   lookup root ((path @ [y]) @ us) \<noteq> None"
                 by cases (auto dest: access_some_lookup)
               then show ?thesis 
-                by (simp add: not_None_eq, blast dest!: lookup_some_append)
+                by (simp, blast dest!: lookup_some_append)
             qed
             finally show ?thesis .
           qed