equal
deleted
inserted
replaced
181 lemma "(\<forall>x. P x \<longrightarrow> Q x) \<Longrightarrow> P y \<Longrightarrow> Q y" |
181 lemma "(\<forall>x. P x \<longrightarrow> Q x) \<Longrightarrow> P y \<Longrightarrow> Q y" |
182 apply guess_all |
182 apply guess_all |
183 apply prop_solver |
183 apply prop_solver |
184 done |
184 done |
185 |
185 |
186 lemma "(\<forall>x. P x \<longrightarrow> Q x) \<Longrightarrow> P z \<Longrightarrow> P y \<Longrightarrow> Q y" |
186 lemma "(\<forall>x. P x \<longrightarrow> Q x) \<Longrightarrow> P z \<Longrightarrow> P y \<Longrightarrow> Q y" |
187 apply (solves \<open>guess_all, prop_solver\<close>) \<comment> \<open>Try it without solve\<close> |
187 apply (solves \<open>guess_all, prop_solver\<close>) \<comment> \<open>Try it without solve\<close> |
188 done |
188 done |
189 |
189 |
190 method guess_ex = |
190 method guess_ex = |
191 (match conclusion in |
191 (match conclusion in |