src/HOL/UNITY/Union.thy
changeset 67613 ce654b0e6d69
parent 63146 f1ecba0272f9
child 69313 b021008c5397
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
    34   where "\<bottom> = mk_program (UNIV, {}, UNIV)"
    34   where "\<bottom> = mk_program (UNIV, {}, UNIV)"
    35 
    35 
    36   (*Characterizes safety properties.  Used with specifying Allowed*)
    36   (*Characterizes safety properties.  Used with specifying Allowed*)
    37 definition
    37 definition
    38   safety_prop :: "'a program set => bool"
    38   safety_prop :: "'a program set => bool"
    39   where "safety_prop X \<longleftrightarrow> SKIP: X & (\<forall>G. Acts G \<subseteq> UNION X Acts --> G \<in> X)"
    39   where "safety_prop X \<longleftrightarrow> SKIP \<in> X \<and> (\<forall>G. Acts G \<subseteq> UNION X Acts \<longrightarrow> G \<in> X)"
    40 
    40 
    41 syntax
    41 syntax
    42   "_JOIN1" :: "[pttrns, 'b set] => 'b set"              ("(3\<Squnion>_./ _)" 10)
    42   "_JOIN1" :: "[pttrns, 'b set] => 'b set"              ("(3\<Squnion>_./ _)" 10)
    43   "_JOIN"  :: "[pttrn, 'a set, 'b set] => 'b set"       ("(3\<Squnion>_\<in>_./ _)" 10)
    43   "_JOIN"  :: "[pttrn, 'a set, 'b set] => 'b set"       ("(3\<Squnion>_\<in>_./ _)" 10)
    44 translations
    44 translations