(* Title: HOL/Corec_Examples/Stream_Processor.thy Author: Andreas Lochbihler, ETH Zuerich Author: Dmitriy Traytel, ETH Zuerich Author: Andrei Popescu, TU Muenchen Copyright 2014, 2016 Stream processors---a syntactic representation of continuous functions on streams. *) section ‹Stream Processors---A Syntactic Representation of Continuous Functions on Streams› theory Stream_Processor imports "HOL-Library.BNF_Corec" "HOL-Library.Stream" begin