tuned -- no need for slightly obscure "local" prefix;
authorwenzelm
Wed, 19 Mar 2014 23:13:45 +0100
changeset 56222 6599c6278545
parent 56221 a8dfbe9f25da
child 56223 7696903b9e61
tuned -- no need for slightly obscure "local" prefix;
src/HOL/Probability/Fin_Map.thy
--- 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