src/HOL/Codatatype/Examples/Infinite_Derivation_Trees/Parallel.thy
changeset 49463 83ac281bcdc2
parent 48975 7f79f94a432c
child 49508 1e205327f059
equal deleted inserted replaced
49462:9ef072c757ca 49463:83ac281bcdc2
       
     1 (*  Title:      HOL/Codatatype/Examples/Infinite_Derivation_Trees/Parallel.thy
       
     2     Author:     Andrei Popescu, TU Muenchen
       
     3     Copyright   2012
       
     4 
       
     5 Parallel composition.
       
     6 *)
       
     7 
       
     8 header {* Parallel Composition *}
       
     9 
     1 theory Parallel 
    10 theory Parallel 
     2 imports Tree
    11 imports Tree
     3 begin
    12 begin
     4 
    13 
     5 
    14