variable name changed
authorhuffman
Tue, 02 Mar 2010 17:20:03 -0800
changeset 35524 a2a59e92b02e
parent 35523 cc57f4a274a3
child 35525 fa231b86cb1e
variable name changed
src/HOLCF/ex/Stream.thy
--- a/src/HOLCF/ex/Stream.thy	Tue Mar 02 16:25:59 2010 -0800
+++ b/src/HOLCF/ex/Stream.thy	Tue Mar 02 17:20:03 2010 -0800
@@ -290,12 +290,12 @@
 
 lemma stream_finite_lemma1: "stream_finite xs ==> stream_finite (x && xs)"
 apply (simp add: stream.finite_def,auto)
-apply (rule_tac x="Suc n" in exI)
+apply (rule_tac x="Suc i" in exI)
 by (simp add: stream_take_lemma4)
 
 lemma stream_finite_lemma2: "[| x ~= UU; stream_finite (x && xs) |] ==> stream_finite xs"
 apply (simp add: stream.finite_def, auto)
-apply (rule_tac x="n" in exI)
+apply (rule_tac x="i" in exI)
 by (erule stream_take_lemma3,simp)
 
 lemma stream_finite_rt_eq: "stream_finite (rt$s) = stream_finite s"