ProgTutorial/Recipes/ExternalSolver.thy
changeset 211 d5accbc67e1b
parent 189 069d525f8f1d
child 346 0fea8b7a14a1
equal deleted inserted replaced
210:db8e302f44c8 211:d5accbc67e1b
     1 theory ExternalSolver
     1 theory ExternalSolver
     2 imports "../Base"
     2 imports "../Base"
     3 begin
     3 begin
     4 
     4 
     5 
     5 
     6 section {* Executing an External Application \label{rec:external}*}
     6 section {* Executing an External Application (TBD) \label{rec:external}*}
     7 
     7 
     8 text {*
     8 text {*
     9   {\bf Problem:}
     9   {\bf Problem:}
    10   You want to use an external application.
    10   You want to use an external application.
    11   \smallskip
    11   \smallskip