equal
deleted
inserted
replaced
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} |