src/HOL/IMP/Abs_Int_ITP/Abs_Int1_ITP.thy
changeset 47818 151d137f1095
parent 47613 e72e44cee6f2
child 52046 bc01725d7918
equal deleted inserted replaced
47817:5d2d63f4363e 47818:151d137f1095
    64 next
    64 next
    65   case Assign thus ?case
    65   case Assign thus ?case
    66     by (fastforce simp: Assign_le  map_acom_Assign intro: aval'_sound in_gamma_update
    66     by (fastforce simp: Assign_le  map_acom_Assign intro: aval'_sound in_gamma_update
    67       split: option.splits del:subsetD)
    67       split: option.splits del:subsetD)
    68 next
    68 next
    69   case Semi thus ?case apply (auto simp: Semi_le map_acom_Semi)
    69   case Seq thus ?case apply (auto simp: Seq_le map_acom_Seq)
    70     by (metis le_post post_map_acom)
    70     by (metis le_post post_map_acom)
    71 next
    71 next
    72   case (If b c1 c2 P)
    72   case (If b c1 c2 P)
    73   then obtain c1' c2' P' where
    73   then obtain c1' c2' P' where
    74       "c' = IF b THEN c1' ELSE c2' {P'}"
    74       "c' = IF b THEN c1' ELSE c2' {P'}"