| changeset 63649 | e690d6f2185b |
| parent 63192 | a742d309afa2 |
| child 64242 | 93c6f0da5c70 |
--- a/src/HOL/Library/Stream.thy Wed Aug 10 09:33:54 2016 +0200 +++ b/src/HOL/Library/Stream.thy Wed Aug 10 14:50:59 2016 +0200 @@ -393,7 +393,7 @@ then show "s = sconst x" proof (coinduction arbitrary: s) case Eq_stream - then have "shd s = x" "sset (stl s) \<subseteq> {x}" by (case_tac [!] s) auto + then have "shd s = x" "sset (stl s) \<subseteq> {x}" by (cases s; auto)+ then have "sset (stl s) = {x}" by (cases "stl s") auto with \<open>shd s = x\<close> show ?case by auto qed