| changeset 58607 | 1f90ea1b4010 |
| parent 58606 | 9c66f7c541fb |
| child 59000 | 6eb0725503fc |
--- a/src/HOL/Probability/Stream_Space.thy Tue Oct 07 10:34:24 2014 +0200 +++ b/src/HOL/Probability/Stream_Space.thy Tue Oct 07 10:48:29 2014 +0200 @@ -4,7 +4,7 @@ theory Stream_Space imports Infinite_Product_Measure - "~~/src/HOL/Datatype_Examples/Stream" + "~~/src/HOL/Library/Stream" begin lemma stream_eq_Stream_iff: "s = x ## t \<longleftrightarrow> (shd s = x \<and> stl s = t)"