src/HOL/Unix/Unix.thy
changeset 46206 d3d62b528487
parent 45671 1c769a2a2421
child 47099 56adbf5bcc82
--- a/src/HOL/Unix/Unix.thy	Sat Jan 14 13:11:32 2012 +0100
+++ b/src/HOL/Unix/Unix.thy	Sat Jan 14 13:22:39 2012 +0100
@@ -1034,7 +1034,7 @@
                   lookup root ((path @ [y]) @ us) \<noteq> None"
                 by cases (auto dest: access_some_lookup)
               then show ?thesis 
-                by (simp, blast dest!: lookup_some_append)
+                by (fastforce dest!: lookup_some_append)
             qed
             finally show ?thesis .
           qed