src/HOL/Unix/Unix.thy
changeset 11809 c9ffdd63dd93
parent 11758 b87aa292f50b
child 11881 b46b1bdbe3f5
--- a/src/HOL/Unix/Unix.thy	Tue Oct 16 17:56:12 2001 +0200
+++ b/src/HOL/Unix/Unix.thy	Tue Oct 16 17:58:13 2001 +0200
@@ -591,7 +591,7 @@
   assume r: "\<And>r x r'. r \<midarrow>x\<rightarrow> r' \<Longrightarrow> Q r \<Longrightarrow>  P x \<Longrightarrow> Q r'"
   assume "root =xs\<Rightarrow> root'"
   thus "Q root \<Longrightarrow> (\<forall>x \<in> set xs. P x) \<Longrightarrow> Q root'" (is "PROP ?P root xs root'")
-  proof (induct ?P root xs root')
+  proof (induct root xs root')
     fix root assume "Q root"
     thus "Q root" .
   next