src/Doc/Eisbach/Manual.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 68484 59793df7f853
equal deleted inserted replaced
67442:f075640b8868 67443:3abf6a722518
   247   prop_solver} becomes capable of solving non-trivial propositional
   247   prop_solver} becomes capable of solving non-trivial propositional
   248   tautologies.
   248   tautologies.
   249 \<close>
   249 \<close>
   250 
   250 
   251     lemmas [intros] =
   251     lemmas [intros] =
   252       conjI  \<comment>  \<open>@{thm conjI}\<close>
   252       conjI  \<comment> \<open>@{thm conjI}\<close>
   253       impI  \<comment>  \<open>@{thm impI}\<close>
   253       impI  \<comment> \<open>@{thm impI}\<close>
   254       disjCI  \<comment>  \<open>@{thm disjCI}\<close>
   254       disjCI  \<comment> \<open>@{thm disjCI}\<close>
   255       iffI  \<comment>  \<open>@{thm iffI}\<close>
   255       iffI  \<comment> \<open>@{thm iffI}\<close>
   256       notI  \<comment>  \<open>@{thm notI}\<close>
   256       notI  \<comment> \<open>@{thm notI}\<close>
   257 
   257 
   258     lemmas [elims] =
   258     lemmas [elims] =
   259       impCE  \<comment>  \<open>@{thm impCE}\<close>
   259       impCE  \<comment> \<open>@{thm impCE}\<close>
   260       conjE  \<comment>  \<open>@{thm conjE}\<close>
   260       conjE  \<comment> \<open>@{thm conjE}\<close>
   261       disjE  \<comment>  \<open>@{thm disjE}\<close>
   261       disjE  \<comment> \<open>@{thm disjE}\<close>
   262 
   262 
   263     lemma "(A \<or> B) \<and> (A \<longrightarrow> C) \<and> (B \<longrightarrow> C) \<longrightarrow> C"
   263     lemma "(A \<or> B) \<and> (A \<longrightarrow> C) \<and> (B \<longrightarrow> C) \<longrightarrow> C"
   264       by prop_solver
   264       by prop_solver
   265 
   265 
   266 
   266