equal
deleted
inserted
replaced
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 |