src/HOL/BNF/Examples/Process.thy
changeset 51804 be6e703908f4
parent 49594 55e798614c45
child 53013 3fbcfa911863
equal deleted inserted replaced
51803:71260347b7e4 51804:be6e703908f4
    11 imports "../BNF"
    11 imports "../BNF"
    12 begin
    12 begin
    13 
    13 
    14 hide_fact (open) Quotient_Product.prod_rel_def
    14 hide_fact (open) Quotient_Product.prod_rel_def
    15 
    15 
    16 codata 'a process =
    16 codatatype 'a process =
    17   isAction: Action (prefOf: 'a) (contOf: "'a process") |
    17   isAction: Action (prefOf: 'a) (contOf: "'a process") |
    18   isChoice: Choice (ch1Of: "'a process") (ch2Of: "'a process")
    18   isChoice: Choice (ch1Of: "'a process") (ch2Of: "'a process")
    19 
    19 
    20 (* Read: prefix of, continuation of, choice 1 of, choice 2 of *)
    20 (* Read: prefix of, continuation of, choice 1 of, choice 2 of *)
    21 
    21