src/HOL/BNF_Examples/Stream_Processor.thy
changeset 57634 efc00b9b8680
parent 57398 882091eb1e9a
child 57641 dc59f147b27d
equal deleted inserted replaced
57633:4ff8c090d580 57634:efc00b9b8680
     1 (*  Title:      HOL/BNF_Examples/Stream_Processor.thy
     1 (*  Title:      HOL/BNF_Examples/Stream_Processor.thy
     2     Author:     Dmitriy Traytel, TU Muenchen
     2     Author:     Dmitriy Traytel, TU Muenchen
     3     Author:     Andrei Popescu, TU Muenchen
     3     Author:     Andrei Popescu, TU Muenchen
     4     Copyright   2014
     4     Copyright   2014
     5 
     5 
     6 Stream processors---a syntactic representation of continuous functions on streams
     6 Stream processors---a syntactic representation of continuous functions on streams.
     7 *)
     7 *)
     8 
     8 
     9 header {* Stream Processors *}
     9 header {* Stream Processors---A Syntactic Representation of Continuous Functions on Streams *}
    10 
    10 
    11 theory Stream_Processor
    11 theory Stream_Processor
    12 imports Stream "~~/src/HOL/Library/BNF_Axiomatization"
    12 imports Stream "~~/src/HOL/Library/BNF_Axiomatization"
    13 begin
    13 begin
    14 
    14