src/HOL/Probability/Fin_Map.thy
changeset 56222 6599c6278545
parent 53374 a14d2a854c02
child 56633 18f50d5f84ef
--- a/src/HOL/Probability/Fin_Map.thy	Wed Mar 19 22:26:27 2014 +0100
+++ b/src/HOL/Probability/Fin_Map.thy	Wed Mar 19 23:13:45 2014 +0100
@@ -545,8 +545,8 @@
   thus "Pi' I S \<in> range ?f" by simp
 next
   fix x and f::"'a \<Rightarrow>\<^sub>F nat"
-  show "\<exists>I S. (\<Pi>' i\<in>domain f. from_nat_into local.basis_proj ((f)\<^sub>F i)) = Pi' I S \<and>
-    finite I \<and> (\<forall>i\<in>I. S i \<in> local.basis_proj)"
+  show "\<exists>I S. (\<Pi>' i\<in>domain f. from_nat_into basis_proj ((f)\<^sub>F i)) = Pi' I S \<and>
+    finite I \<and> (\<forall>i\<in>I. S i \<in> basis_proj)"
     using assms by (auto intro: from_nat_into)
 qed