src/HOL/Induct/LList.thy
changeset 15944 9b00875e21f7
parent 15481 fc075ae929e4
child 16417 9bc16273c2d4
--- a/src/HOL/Induct/LList.thy	Mon May 09 16:02:45 2005 +0200
+++ b/src/HOL/Induct/LList.thy	Mon May 09 16:38:56 2005 +0200
@@ -865,7 +865,8 @@
        in llist_equalityI)
  apply (rule rangeI)
 apply (safe)
-apply (simplesubst iterates, simp)  --{*two redexes*}
+apply (subst (1 2) iterates)
+apply simp 
 done
 
 subsubsection{* Two proofs that @{text lmap} distributes over lappend *}