src/HOL/Unix/Unix.thy
changeset 20503 503ac4c5ef91
parent 20321 b7c0bf788f50
child 21001 408f3a1cef2e
--- a/src/HOL/Unix/Unix.thy	Mon Sep 11 14:35:30 2006 +0200
+++ b/src/HOL/Unix/Unix.thy	Mon Sep 11 21:35:19 2006 +0200
@@ -657,7 +657,7 @@
 
 lemma can_exec_snocD: "can_exec root (xs @ [y])
     \<Longrightarrow> \<exists>root' root''. root =xs\<Rightarrow> root' \<and> root' \<midarrow>y\<rightarrow> root''"
-proof (induct xs fixing: root)
+proof (induct xs arbitrary: root)
   case Nil
   then show ?case
     by (simp add: can_exec_def transitions_nil_eq transitions_cons_eq)