src/HOL/HOLCF/IOA/ABP/Correctness.thy
changeset 58880 0baae4311a9f
parent 51717 9e7d1c139569
child 61032 b57df8eecad6
equal deleted inserted replaced
58879:143c85e3cdb5 58880:0baae4311a9f
     1 (*  Title:      HOL/HOLCF/IOA/ABP/Correctness.thy
     1 (*  Title:      HOL/HOLCF/IOA/ABP/Correctness.thy
     2     Author:     Olaf Müller
     2     Author:     Olaf Müller
     3 *)
     3 *)
     4 
     4 
     5 header {* The main correctness proof: System_fin implements System *}
     5 section {* The main correctness proof: System_fin implements System *}
     6 
     6 
     7 theory Correctness
     7 theory Correctness
     8 imports IOA Env Impl Impl_finite
     8 imports IOA Env Impl Impl_finite
     9 begin
     9 begin
    10 
    10