src/HOLCF/Library/Stream.thy
changeset 40025 876689e6bbdf
parent 40002 c5b5f7a3a3b1
child 40213 b63e966564da
--- a/src/HOLCF/Library/Stream.thy	Sat Oct 16 14:41:11 2010 -0700
+++ b/src/HOLCF/Library/Stream.thy	Sat Oct 16 15:26:30 2010 -0700
@@ -265,7 +265,7 @@
  apply (simp add: stream.bisim_def,clarsimp)
  apply (drule spec, drule spec, drule (1) mp)
  apply (case_tac "x", simp)
- apply (case_tac "x'", simp)
+ apply (case_tac "y", simp)
 by auto