src/HOL/SMT.thy
changeset 55049 327eafb594ba
parent 55007 0c07990363a3
child 56046 683148f3ae48
equal deleted inserted replaced
55043:acefda71629b 55049:327eafb594ba
   202 Each SMT solver provides several commandline options to tweak its
   202 Each SMT solver provides several commandline options to tweak its
   203 behaviour.  They can be passed to the solver by setting the following
   203 behaviour.  They can be passed to the solver by setting the following
   204 options.
   204 options.
   205 *}
   205 *}
   206 
   206 
   207 declare [[ cvc3_options = "", remote_cvc3_options = "" ]]
   207 declare [[ cvc3_options = "" ]]
   208 declare [[ yices_options = "" ]]
   208 declare [[ yices_options = "" ]]
   209 declare [[ z3_options = "", remote_z3_options = "" ]]
   209 declare [[ z3_options = "" ]]
   210 
   210 
   211 text {*
   211 text {*
   212 Enable the following option to use built-in support for datatypes and
   212 Enable the following option to use built-in support for datatypes and
   213 records.  Currently, this is only implemented for Z3 running in oracle
   213 records.  Currently, this is only implemented for Z3 running in oracle
   214 mode.
   214 mode.