src/HOL/UNITY/Simple/Reachability.thy
changeset 46911 6d2a2f0e904e
parent 46008 c296c75f4cf4
child 62390 842917225d56
equal deleted inserted replaced
46910:3e068ef04b42 46911:6d2a2f0e904e
   317    apply (blast intro: Stable_INT Stable_reachable_EQ_R_AND_nmsg_0
   317    apply (blast intro: Stable_INT Stable_reachable_EQ_R_AND_nmsg_0
   318                     Leadsto_reachability_AND_nmsg_0)+
   318                     Leadsto_reachability_AND_nmsg_0)+
   319 done
   319 done
   320 
   320 
   321 lemma LeadsTo_final: "F \<in> UNIV LeadsTo final"
   321 lemma LeadsTo_final: "F \<in> UNIV LeadsTo final"
   322 apply (case_tac "E={}")
   322 apply (cases "E={}")
   323  apply (rule_tac [2] LeadsTo_final_E_NOT_empty)
   323  apply (rule_tac [2] LeadsTo_final_E_NOT_empty)
   324 apply (rule LeadsTo_final_E_empty, auto)
   324 apply (rule LeadsTo_final_E_empty, auto)
   325 done
   325 done
   326 
   326 
   327 (* ------------------------------------ *)
   327 (* ------------------------------------ *)
   359               (- {} \<union> nmsg_eq 0 (v,w)))")
   359               (- {} \<union> nmsg_eq 0 (v,w)))")
   360 apply blast+
   360 apply blast+
   361 done
   361 done
   362 
   362 
   363 lemma Stable_final: "F \<in> Stable final"
   363 lemma Stable_final: "F \<in> Stable final"
   364 apply (case_tac "E={}")
   364 apply (cases "E={}")
   365  prefer 2 apply (blast intro: Stable_final_E_NOT_empty)
   365  prefer 2 apply (blast intro: Stable_final_E_NOT_empty)
   366 apply (blast intro: Stable_final_E_empty)
   366 apply (blast intro: Stable_final_E_empty)
   367 done
   367 done
   368 
   368 
   369 end
   369 end