src/HOL/Hoare_Parallel/RG_Com.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58884 be4d203d35b3
equal deleted inserted replaced
58309:a09ec6daaa19 58310:91ea607a34d8
    10 of states.  Syntax of commands @{text com} and parallel commands
    10 of states.  Syntax of commands @{text com} and parallel commands
    11 @{text par_com}. *}
    11 @{text par_com}. *}
    12 
    12 
    13 type_synonym 'a bexp = "'a set"
    13 type_synonym 'a bexp = "'a set"
    14 
    14 
    15 datatype_new 'a com = 
    15 datatype 'a com = 
    16     Basic "'a \<Rightarrow>'a"
    16     Basic "'a \<Rightarrow>'a"
    17   | Seq "'a com" "'a com"
    17   | Seq "'a com" "'a com"
    18   | Cond "'a bexp" "'a com" "'a com"         
    18   | Cond "'a bexp" "'a com" "'a com"         
    19   | While "'a bexp" "'a com"       
    19   | While "'a bexp" "'a com"       
    20   | Await "'a bexp" "'a com"                 
    20   | Await "'a bexp" "'a com"