src/HOL/SMT2.thy
changeset 57237 bc51864c2ac4
parent 57230 ec5ff6bb2a92
child 57239 a40edeaa01b1
equal deleted inserted replaced
57236:2eb14982cd29 57237:bc51864c2ac4
   160 text {*
   160 text {*
   161 The option @{text smt2_solver} can be used to change the target SMT
   161 The option @{text smt2_solver} can be used to change the target SMT
   162 solver.  The possible values can be obtained from the @{text smt2_status}
   162 solver.  The possible values can be obtained from the @{text smt2_status}
   163 command.
   163 command.
   164 
   164 
   165 Due to licensing restrictions, Yices and Z3 are not installed/enabled
   165 Due to licensing restrictions, Z3 is not enabled by default.  Z3 is free
   166 by default.  Z3 is free for non-commercial applications and can be enabled
   166 for non-commercial applications and can be enabled by setting Isabelle
   167 by setting Isabelle system option @{text z3_non_commercial} to @{text yes}.
   167 system option @{text z3_non_commercial} to @{text yes}.
   168 *}
   168 *}
   169 
   169 
   170 declare [[smt2_solver = z3]]
   170 declare [[smt2_solver = z3]]
   171 
   171 
   172 text {*
   172 text {*
   198 behaviour.  They can be passed to the solver by setting the following
   198 behaviour.  They can be passed to the solver by setting the following
   199 options.
   199 options.
   200 *}
   200 *}
   201 
   201 
   202 declare [[cvc3_new_options = ""]]
   202 declare [[cvc3_new_options = ""]]
   203 declare [[yices_new_options = ""]]
       
   204 declare [[z3_new_options = ""]]
   203 declare [[z3_new_options = ""]]
   205 
   204 
   206 text {*
   205 text {*
   207 The SMT method provides an inference mechanism to detect simple triggers
   206 The SMT method provides an inference mechanism to detect simple triggers
   208 in quantified formulas, which might increase the number of problems
   207 in quantified formulas, which might increase the number of problems