src/HOL/HOLCF/FOCUS/Fstream.thy
changeset 58880 0baae4311a9f
parent 45049 13efaee97111
child 61998 b66d2ca1f907
equal deleted inserted replaced
58879:143c85e3cdb5 58880:0baae4311a9f
     4 FOCUS streams (with lifted elements).
     4 FOCUS streams (with lifted elements).
     5 
     5 
     6 TODO: integrate Fstreams.thy
     6 TODO: integrate Fstreams.thy
     7 *)
     7 *)
     8 
     8 
     9 header {* FOCUS flat streams *}
     9 section {* FOCUS flat streams *}
    10 
    10 
    11 theory Fstream
    11 theory Fstream
    12 imports "~~/src/HOL/HOLCF/Library/Stream"
    12 imports "~~/src/HOL/HOLCF/Library/Stream"
    13 begin
    13 begin
    14 
    14