src/HOL/Hoare_Parallel/RG_Tran.thy
changeset 67613 ce654b0e6d69
parent 67443 3abf6a722518
child 71989 bad75618fb82
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
    26   ctran :: "('a conf \<times> 'a conf) set"
    26   ctran :: "('a conf \<times> 'a conf) set"
    27   and ctran' :: "'a conf \<Rightarrow> 'a conf \<Rightarrow> bool"   ("_ -c\<rightarrow> _" [81,81] 80)
    27   and ctran' :: "'a conf \<Rightarrow> 'a conf \<Rightarrow> bool"   ("_ -c\<rightarrow> _" [81,81] 80)
    28   and ctrans :: "'a conf \<Rightarrow> 'a conf \<Rightarrow> bool"   ("_ -c*\<rightarrow> _" [81,81] 80)
    28   and ctrans :: "'a conf \<Rightarrow> 'a conf \<Rightarrow> bool"   ("_ -c*\<rightarrow> _" [81,81] 80)
    29 where
    29 where
    30   "P -c\<rightarrow> Q \<equiv> (P,Q) \<in> ctran"
    30   "P -c\<rightarrow> Q \<equiv> (P,Q) \<in> ctran"
    31 | "P -c*\<rightarrow> Q \<equiv> (P,Q) \<in> ctran^*"
    31 | "P -c*\<rightarrow> Q \<equiv> (P,Q) \<in> ctran\<^sup>*"
    32 
    32 
    33 | Basic:  "(Some(Basic f), s) -c\<rightarrow> (None, f s)"
    33 | Basic:  "(Some(Basic f), s) -c\<rightarrow> (None, f s)"
    34 
    34 
    35 | Seq1:   "(Some P0, s) -c\<rightarrow> (None, t) \<Longrightarrow> (Some(Seq P0 P1), s) -c\<rightarrow> (Some P1, t)"
    35 | Seq1:   "(Some P0, s) -c\<rightarrow> (None, t) \<Longrightarrow> (Some(Seq P0 P1), s) -c\<rightarrow> (Some P1, t)"
    36 
    36