src/ZF/UNITY/WFair.thy
changeset 61798 27f3c10b0b50
parent 61392 331be2820f90
child 65449 c82e63b11b8b
--- a/src/ZF/UNITY/WFair.thy	Mon Dec 07 10:19:30 2015 +0100
+++ b/src/ZF/UNITY/WFair.thy	Mon Dec 07 10:23:50 2015 +0100
@@ -283,7 +283,7 @@
 lemma leadsTo_Union_distrib: "(F \<in> \<Union>(S) \<longmapsto> B) \<longleftrightarrow>  (\<forall>A \<in> S. F \<in> A \<longmapsto> B) & F \<in> program & st_set(B)"
 by (blast dest: leadsToD2 intro: leadsTo_Union leadsTo_weaken_L)
 
-text\<open>Set difference: maybe combine with @{text leadsTo_weaken_L}??\<close>
+text\<open>Set difference: maybe combine with \<open>leadsTo_weaken_L\<close>??\<close>
 lemma leadsTo_Diff:
      "[| F: (A-B) \<longmapsto> C; F \<in> B \<longmapsto> C; st_set(C) |]
       ==> F \<in> A \<longmapsto> C"