src/ZF/ex/Limit.thy
changeset 15481 fc075ae929e4
parent 14171 0cab06e3bbd0
child 16417 9bc16273c2d4
--- a/src/ZF/ex/Limit.thy	Sun Jan 30 20:48:50 2005 +0100
+++ b/src/ZF/ex/Limit.thy	Tue Feb 01 18:01:57 2005 +0100
@@ -1242,13 +1242,13 @@
 apply (erule chain_mkcpo)
 done
 
-lemma subcpo_Dinf:
-    "emb_chain(DD,ee) ==> subcpo(Dinf(DD,ee),iprod(DD))"
+lemma subcpo_Dinf: "emb_chain(DD,ee) ==> subcpo(Dinf(DD,ee),iprod(DD))"
 apply (simp add: Dinf_def)
 apply (rule subcpo_mkcpo)
 apply (simp add: Dinf_def [symmetric])
 apply (rule ballI)
-apply (subst lub_iprod)
+apply (simplesubst lub_iprod)
+  --{*Subst would rewrite the lhs. We want to change the rhs.*}
 apply (assumption | rule chain_Dinf emb_chain_cpo)+
 apply simp
 apply (subst Rp_cont [THEN cont_lub])
@@ -1688,7 +1688,8 @@
 apply (rule_tac i = "succ (na) " and j = n in nat_linear_le)
    apply blast
   apply assumption
- apply (subst eps_split_right_le)
+ apply (simplesubst eps_split_right_le)
+    --{*Subst would rewrite the lhs. We want to change the rhs.*}
        prefer 2 apply assumption
       apply simp
      apply (assumption | rule add_le_self nat_0I nat_succI)+