src/Doc/Prog_Prove/Logic.thy
changeset 63414 beb987127d0f
parent 62223 c82c7b78b509
child 63935 aa1fe1103ab8
equal deleted inserted replaced
63413:9fe2d9dc095e 63414:beb987127d0f
   307 
   307 
   308 If you want to try all of the above automatic proof methods you simply type
   308 If you want to try all of the above automatic proof methods you simply type
   309 \begin{isabelle}
   309 \begin{isabelle}
   310 \isacom{try}
   310 \isacom{try}
   311 \end{isabelle}
   311 \end{isabelle}
   312 You can also add specific simplification and introduction rules:
   312 There is also a lightweight variant \isacom{try0} that does not call
       
   313 sledgehammer. If desired, specific simplification and introduction rules
       
   314 can be added:
   313 \begin{isabelle}
   315 \begin{isabelle}
   314 \isacom{try} @{text"simp: \<dots> intro: \<dots>"}
   316 \isacom{try0} @{text"simp: \<dots> intro: \<dots>"}
   315 \end{isabelle}
   317 \end{isabelle}
   316 There is also a lightweight variant \isacom{try0} that does not call
       
   317 sledgehammer.
       
   318 
   318 
   319 \section{Single Step Proofs}
   319 \section{Single Step Proofs}
   320 
   320 
   321 Although automation is nice, it often fails, at least initially, and you need
   321 Although automation is nice, it often fails, at least initially, and you need
   322 to find out why. When @{text fastforce} or @{text blast} simply fail, you have
   322 to find out why. When @{text fastforce} or @{text blast} simply fail, you have