src/HOLCF/ex/Stream.thy
changeset 35215 a03462cbf86f
parent 35174 e15040ae75d7
child 35443 2e0f9516947e
--- a/src/HOLCF/ex/Stream.thy	Thu Feb 18 12:36:09 2010 -0800
+++ b/src/HOLCF/ex/Stream.thy	Thu Feb 18 13:29:59 2010 -0800
@@ -358,8 +358,7 @@
 by (drule stream_finite_lemma1,auto)
 
 lemma slen_less_1_eq: "(#x < Fin (Suc 0)) = (x = \<bottom>)"
-by (rule stream.casedist [of x], auto simp del: iSuc_Fin
-    simp add: Fin_0 iSuc_Fin[THEN sym] i0_iless_iSuc iSuc_mono)
+by (rule stream.casedist [of x], auto simp add: Fin_0 iSuc_Fin[THEN sym])
 
 lemma slen_empty_eq: "(#x = 0) = (x = \<bottom>)"
 by (rule stream.casedist [of x], auto)