src/ZF/Univ.thy
changeset 61798 27f3c10b0b50
parent 60770 240563fbf41d
child 69593 3dda49e08b9d
--- a/src/ZF/Univ.thy	Mon Dec 07 10:19:30 2015 +0100
+++ b/src/ZF/Univ.thy	Mon Dec 07 10:23:50 2015 +0100
@@ -77,7 +77,7 @@
 apply (subst Vfrom)
 apply (subst Vfrom, rule subset_refl [THEN Un_mono])
 apply (rule UN_least)
-txt\<open>expand @{text "rank(x1) = (\<Union>y\<in>x1. succ(rank(y)))"} in assumptions\<close>
+txt\<open>expand \<open>rank(x1) = (\<Union>y\<in>x1. succ(rank(y)))\<close> in assumptions\<close>
 apply (erule rank [THEN equalityD1, THEN subsetD, THEN UN_E])
 apply (rule subset_trans)
 apply (erule_tac [2] UN_upper)
@@ -748,7 +748,7 @@
      "[| f: W -||> univ(A);  W \<subseteq> univ(A) |] ==> f \<in> univ(A)"
 by (erule FiniteFun_univ [THEN subsetD], assumption)
 
-text\<open>Remove @{text "\<subseteq>"} from the rule above\<close>
+text\<open>Remove \<open>\<subseteq>\<close> from the rule above\<close>
 lemmas FiniteFun_in_univ' = FiniteFun_in_univ [OF _ subsetI]