CookBook/Recipes/ExternalSolver.thy
changeset 81 8fda6b452f28
parent 79 a53c7810e38b
child 83 0fb5f91d5109
equal deleted inserted replaced
80:95e9c4556221 81:8fda6b452f28
     1 theory ExternalSolver
     1 theory ExternalSolver
     2 imports "../Base"
     2 imports "../Base"
     3 begin
     3 begin
     4 
     4 
     5 section {* Using an External Solver *} 
     5 section {* Using an External Solver\label{rec:external} *} 
     6 
     6 
     7 text {*
     7 text {*
     8   {\bf Problem:}
     8   {\bf Problem:}
     9   You want to use an external solver, because the solver might be more efficient 
     9   You want to use an external solver, because the solver might be more efficient 
    10   for deciding a certain class of formulae than Isabelle tactics.
    10   for deciding a certain class of formulae than Isabelle tactics.