equal
deleted
inserted
replaced
1 (* Title: HOL/Library/Linear_Temporal_Logic_on_Streams.thy |
1 (* Title: HOL/Library/Linear_Temporal_Logic_on_Streams.thy |
2 Author: Andrei Popescu, TU Muenchen |
2 Author: Andrei Popescu, TU Muenchen |
3 Author: Dmitriy Traytel, TU Muenchen |
3 Author: Dmitriy Traytel, TU Muenchen |
4 *) |
4 *) |
5 |
5 |
6 header {* Linear Temporal Logic on Streams *} |
6 section {* Linear Temporal Logic on Streams *} |
7 |
7 |
8 theory Linear_Temporal_Logic_on_Streams |
8 theory Linear_Temporal_Logic_on_Streams |
9 imports Stream Sublist |
9 imports Stream Sublist |
10 begin |
10 begin |
11 |
11 |