src/ZF/UNITY/Distributor.thy
changeset 59788 6f7b6adac439
parent 46823 57bf0cecb366
child 60770 240563fbf41d
--- a/src/ZF/UNITY/Distributor.thy	Mon Mar 23 19:43:03 2015 +0100
+++ b/src/ZF/UNITY/Distributor.thy	Mon Mar 23 21:05:17 2015 +0100
@@ -131,7 +131,7 @@
 apply (subgoal_tac "length (s ` iIn) \<in> nat")
 apply typecheck
 apply (subgoal_tac "m \<in> nat")
-apply (drule_tac x = "nth(m, s`iIn) " and P = "%elt. ?X (elt) \<longrightarrow> elt<Nclients" in bspec)
+apply (drule_tac x = "nth(m, s`iIn) " and P = "%elt. X (elt) \<longrightarrow> elt<Nclients" for X in bspec)
 apply (simp add: ltI)
 apply (simp_all add: Ord_mem_iff_lt)
 apply (blast dest: ltD)