diff -r f7c00119e6e7 -r ca53150406c9 src/HOL/Library/Stream.thy --- a/src/HOL/Library/Stream.thy Sat Nov 14 18:37:49 2015 +0100 +++ b/src/HOL/Library/Stream.thy Sun Nov 15 12:39:51 2015 +0100 @@ -68,12 +68,18 @@ subsection \set of streams with elements in some fixed set\ +context + notes [[inductive_defs]] +begin + coinductive_set streams :: "'a set \ 'a stream set" for A :: "'a set" where Stream[intro!, simp, no_atp]: "\a \ A; s \ streams A\ \ a ## s \ streams A" +end + lemma in_streams: "stl s \ streams S \ shd s \ S \ s \ streams S" by (cases s) auto