src/HOL/HOLCF/IOA/meta_theory/IOA.thy
changeset 40774 0437dbc127b3
parent 35174 e15040ae75d7
child 40945 b8703f63bfb2
equal deleted inserted replaced
40773:6c12f5e24e34 40774:0437dbc127b3
       
     1 (*  Title:      HOLCF/IOA/meta_theory/IOA.thy
       
     2     Author:     Olaf Müller
       
     3 *)
       
     4 
       
     5 header {* The theory of I/O automata in HOLCF *}
       
     6 
       
     7 theory IOA
       
     8 imports SimCorrectness Compositionality Deadlock
       
     9 begin
       
    10 
       
    11 end