doc-src/TutorialI/CTL/PDL.thy
changeset 12815 1f073030b97a
parent 12631 7648ac4a6b95
child 17914 99ead7a7eb42
equal deleted inserted replaced
12814:2f5edb146f7e 12815:1f073030b97a
   172 @{text auto} augmented with the lemma as a simplification rule.
   172 @{text auto} augmented with the lemma as a simplification rule.
   173 *}
   173 *}
   174 
   174 
   175 theorem "mc f = {s. s \<Turnstile> f}"
   175 theorem "mc f = {s. s \<Turnstile> f}"
   176 apply(induct_tac f)
   176 apply(induct_tac f)
   177 apply(auto simp add:EF_lemma)
   177 apply(auto simp add: EF_lemma)
   178 done
   178 done
   179 
   179 
   180 text{*
   180 text{*
   181 \begin{exercise}
   181 \begin{exercise}
   182 @{term AX} has a dual operator @{term EN} 
   182 @{term AX} has a dual operator @{term EN}