doc-src/TutorialI/CTL/CTL.thy
changeset 9992 4281ccea43f0
parent 9958 67f2920862c7
child 10000 fe6ffa46266f
equal deleted inserted replaced
9991:fdead18501ca 9992:4281ccea43f0
   140 apply(rule_tac x = "path s P" in exI);
   140 apply(rule_tac x = "path s P" in exI);
   141 apply(simp);
   141 apply(simp);
   142 apply(intro strip);
   142 apply(intro strip);
   143 apply(induct_tac i);
   143 apply(induct_tac i);
   144  apply(simp);
   144  apply(simp);
   145  apply(fast intro:selectI2EX);
   145  apply(fast intro:someI2EX);
   146 apply(simp);
   146 apply(simp);
   147 apply(rule selectI2EX);
   147 apply(rule someI2EX);
   148  apply(blast);
   148  apply(blast);
   149 apply(rule selectI2EX);
   149 apply(rule someI2EX);
   150  apply(blast);
   150  apply(blast);
   151 by(blast);
   151 by(blast);
   152 
   152 
   153 lemma seq_lemma:
   153 lemma seq_lemma:
   154 "\<lbrakk> P s; \<forall> s. P s \<longrightarrow> (\<exists> t. (s,t)\<in>M \<and> P t) \<rbrakk> \<Longrightarrow>
   154 "\<lbrakk> P s; \<forall> s. P s \<longrightarrow> (\<exists> t. (s,t)\<in>M \<and> P t) \<rbrakk> \<Longrightarrow>
   160 apply(rule_tac x = "nat_rec s (\<lambda>n t. SOME u. (t,u)\<in>M \<and> P u)" in exI);
   160 apply(rule_tac x = "nat_rec s (\<lambda>n t. SOME u. (t,u)\<in>M \<and> P u)" in exI);
   161 apply(simp);
   161 apply(simp);
   162 apply(intro strip);
   162 apply(intro strip);
   163 apply(induct_tac i);
   163 apply(induct_tac i);
   164  apply(simp);
   164  apply(simp);
   165  apply(fast intro:selectI2EX);
   165  apply(fast intro:someI2EX);
   166 apply(simp);
   166 apply(simp);
   167 apply(rule selectI2EX);
   167 apply(rule someI2EX);
   168  apply(blast);
   168  apply(blast);
   169 apply(rule selectI2EX);
   169 apply(rule someI2EX);
   170  apply(blast);
   170  apply(blast);
   171 by(blast);
   171 by(blast);
   172 
   172 
   173 theorem AF_subset_lfp:
   173 theorem AF_subset_lfp:
   174 "{s. \<forall> p \<in> Paths s. \<exists> i. p i \<in> A} \<subseteq> lfp(af A)";
   174 "{s. \<forall> p \<in> Paths s. \<exists> i. p i \<in> A} \<subseteq> lfp(af A)";