src/HOL/Tools/SMT/smt_systems.ML
author desharna
Wed, 22 Jun 2022 14:52:27 +0200
changeset 75585 a789c5732f7a
parent 75339 d9bb81999d2c
child 75806 2b106aae897c
permissions -rw-r--r--
merged
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
     1
(*  Title:      HOL/Tools/SMT/smt_systems.ML
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     2
    Author:     Sascha Boehme, TU Muenchen
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     3
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     4
Setup SMT solvers.
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     5
*)
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     6
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
     7
signature SMT_SYSTEMS =
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
     8
sig
59960
372ddff01244 updated SMT module and Sledgehammer to fully open source Z3
blanchet
parents: 59035
diff changeset
     9
  val cvc4_extensions: bool Config.T
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    10
  val z3_extensions: bool Config.T
57229
blanchet
parents: 57210
diff changeset
    11
end;
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    12
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    13
structure SMT_Systems: SMT_SYSTEMS =
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    14
struct
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    15
75029
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    16
val mashN = "mash"
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    17
val mepoN = "mepo"
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    18
val meshN = "mesh"
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    19
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    20
(* helper functions *)
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    21
72478
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
    22
fun check_tool var () =
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
    23
  (case getenv var of
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
    24
    "" => NONE
72479
7d0861af3cb0 proper support for Windows exe;
wenzelm
parents: 72478
diff changeset
    25
  | s =>
7d0861af3cb0 proper support for Windows exe;
wenzelm
parents: 72478
diff changeset
    26
      if File.is_file (Path.variable var |> Path.expand |> Path.platform_exe)
7d0861af3cb0 proper support for Windows exe;
wenzelm
parents: 72478
diff changeset
    27
      then SOME [s] else NONE);
72478
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
    28
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    29
fun make_avail name () = getenv (name ^ "_SOLVER") <> ""
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    30
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    31
fun make_command name () = [getenv (name ^ "_SOLVER")]
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    32
70327
c04d4951a155 handle timeouts gracefully in 'smt' proof method (patch due to Mathias Fleury)
blanchet
parents: 69593
diff changeset
    33
fun outcome_of unsat sat unknown timeout solver_name line =
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    34
  if String.isPrefix unsat line then SMT_Solver.Unsat
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    35
  else if String.isPrefix sat line then SMT_Solver.Sat
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    36
  else if String.isPrefix unknown line then SMT_Solver.Unknown
70327
c04d4951a155 handle timeouts gracefully in 'smt' proof method (patch due to Mathias Fleury)
blanchet
parents: 69593
diff changeset
    37
  else if String.isPrefix timeout line then SMT_Solver.Time_Out
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    38
  else raise SMT_Failure.SMT (SMT_Failure.Other_Failure ("Solver " ^ quote solver_name ^
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    39
    " failed -- enable tracing using the " ^ quote (Config.name_of SMT_Config.trace) ^
56094
2adbc6e4cd8f let exception pass through in debug mode
blanchet
parents: 56091
diff changeset
    40
    " option for details"))
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    41
73104
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    42
(* When used with bitvectors, CVC4 can produce error messages like:
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    43
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    44
$ISABELLE_TMP_PREFIX/... No set-logic command was given before this point.
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    45
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    46
These message should be ignored.
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    47
*)
60201
90e88e521e0e made CVC4 support work also without unsat cores
blanchet
parents: 59960
diff changeset
    48
fun is_blank_or_error_line "" = true
73104
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    49
  | is_blank_or_error_line s =
6520d59fbdd7 ignore error messages produced by CVC4 when generating BV
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 72667
diff changeset
    50
  String.isPrefix "(error " s orelse String.isPrefix (getenv "ISABELLE_TMP_PREFIX") s
60201
90e88e521e0e made CVC4 support work also without unsat cores
blanchet
parents: 59960
diff changeset
    51
57239
a40edeaa01b1 don't ask proof-disabled solvers to do proofs
blanchet
parents: 57237
diff changeset
    52
fun on_first_line test_outcome solver_name lines =
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    53
  let
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    54
    val split_first = (fn [] => ("", []) | l :: ls => (l, ls))
67522
9e712280cc37 clarified take/drop/chop prefix/suffix;
wenzelm
parents: 67405
diff changeset
    55
    val (l, ls) = split_first (drop_prefix is_blank_or_error_line lines)
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    56
  in (test_outcome solver_name l, ls) end
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    57
57704
c0da3fc313e3 Basic support for the SMT prover veriT.
fleury
parents: 57240
diff changeset
    58
fun on_first_non_unsupported_line test_outcome solver_name lines =
67405
e9ab4ad7bd15 uniform use of Standard ML op-infix -- eliminated warnings;
wenzelm
parents: 67399
diff changeset
    59
  on_first_line test_outcome solver_name (filter (curry (op <>) "unsupported") lines)
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
    60
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    61
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    62
(* CVC4 *)
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    63
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 69205
diff changeset
    64
val cvc4_extensions = Attrib.setup_config_bool \<^binding>\<open>cvc4_extensions\<close> (K false)
58360
dee1fd1cc631 added interface for CVC4 extensions
blanchet
parents: 58061
diff changeset
    65
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    66
local
73388
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    67
  fun cvc4_options ctxt =
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    68
    ["--no-stats",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    69
     "--random-seed=" ^ string_of_int (Config.get ctxt SMT_Config.random_seed),
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    70
     "--lang=smt2"] @
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    71
    (case SMT_Config.get_timeout ctxt of
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    72
      NONE => []
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
    73
    | SOME t => ["--tlimit", string_of_int (Time.toMilliseconds t)])
58360
dee1fd1cc631 added interface for CVC4 extensions
blanchet
parents: 58061
diff changeset
    74
dee1fd1cc631 added interface for CVC4 extensions
blanchet
parents: 58061
diff changeset
    75
  fun select_class ctxt =
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    76
    if Config.get ctxt cvc4_extensions then
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    77
      if Config.get ctxt SMT_Config.higher_order then
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    78
        CVC4_Interface.hosmtlib_cvc4C
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    79
      else
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    80
        CVC4_Interface.smtlib_cvc4C
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    81
    else
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    82
      if Config.get ctxt SMT_Config.higher_order then
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    83
        SMTLIB_Interface.hosmtlibC
74817
1fd8705503b4 generate problems with correct logic for veriT
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74691
diff changeset
    84
      else if Config.get ctxt SMT_Config.native_bv then
1fd8705503b4 generate problems with correct logic for veriT
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74691
diff changeset
    85
        SMTLIB_Interface.bvsmlibC
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    86
      else
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
    87
        SMTLIB_Interface.smtlibC
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    88
in
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    89
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
    90
val cvc4: SMT_Solver.solver_config = {
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    91
  name = "cvc4",
58360
dee1fd1cc631 added interface for CVC4 extensions
blanchet
parents: 58061
diff changeset
    92
  class = select_class,
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    93
  avail = make_avail "CVC4",
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    94
  command = make_command "CVC4",
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
    95
  options = cvc4_options,
59015
627a93f67182 parse CVC4 unsat cores
blanchet
parents: 58496
diff changeset
    96
  smt_options = [(":produce-unsat-cores", "true")],
75029
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    97
  good_slices =
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
    98
    (* FUDGE *)
75339
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
    99
    [((1, 512, meshN), ["--full-saturate-quant", "--inst-when=full-last-call", "--inst-no-entail", "--term-db-mode=relevant", "--multi-trigger-linear"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   100
     ((1, 64, meshN), ["--decision=internal", "--simplification=none", "--full-saturate-quant"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   101
     ((1, 1024, meshN), ["--relevant-triggers", "--full-saturate-quant"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   102
     ((1, 256, mepoN), ["--trigger-sel=max", "--full-saturate-quant"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   103
     ((1, 32, meshN), ["--term-db-mode=relevant", "--full-saturate-quant"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   104
     ((1, 128, meshN), ["--no-e-matching", "--full-saturate-quant"]),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   105
     ((1, 256, meshN), ["--finite-model-find", "--fmf-inst-engine"])],
70327
c04d4951a155 handle timeouts gracefully in 'smt' proof method (patch due to Mathias Fleury)
blanchet
parents: 69593
diff changeset
   106
  outcome = on_first_line (outcome_of "unsat" "sat" "unknown" "timeout"),
59015
627a93f67182 parse CVC4 unsat cores
blanchet
parents: 58496
diff changeset
   107
  parse_proof = SOME (K CVC4_Proof_Parse.parse_proof),
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
   108
  replay = NONE }
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
   109
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
   110
end
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
   111
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   112
57704
c0da3fc313e3 Basic support for the SMT prover veriT.
fleury
parents: 57240
diff changeset
   113
(* veriT *)
c0da3fc313e3 Basic support for the SMT prover veriT.
fleury
parents: 57240
diff changeset
   114
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   115
local
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   116
  fun select_class ctxt =
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   117
    if Config.get ctxt SMT_Config.higher_order then
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   118
      SMTLIB_Interface.hosmtlibC
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   119
    else
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   120
      SMTLIB_Interface.smtlibC
73388
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   121
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   122
  fun veriT_options ctxt =
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   123
   ["--proof-with-sharing",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   124
    "--proof-define-skolems",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   125
    "--proof-prune",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   126
    "--proof-merge",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   127
    "--disable-print-success",
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   128
    "--disable-banner"] @
74476
6424c54157d9 added timeout to veriT
desharna
parents: 74048
diff changeset
   129
    Verit_Proof.veriT_current_strategy (Context.Proof ctxt) @
6424c54157d9 added timeout to veriT
desharna
parents: 74048
diff changeset
   130
    (case SMT_Config.get_timeout ctxt of
6424c54157d9 added timeout to veriT
desharna
parents: 74048
diff changeset
   131
      NONE => []
74553
3ec9cafab990 proper veriT --max-time option
desharna
parents: 74476
diff changeset
   132
    | SOME t => ["--max-time=" ^ string_of_int (Time.toMilliseconds t)])
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   133
in
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   134
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   135
val veriT: SMT_Solver.solver_config = {
59035
3a2153676705 renamed 'veriT' to 'verit', to stick to all-lowercase rule for prover names
blanchet
parents: 59015
diff changeset
   136
  name = "verit",
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   137
  class = select_class,
72478
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
   138
  avail = is_some o check_tool "ISABELLE_VERIT",
b452242dce36 proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
wenzelm
parents: 72458
diff changeset
   139
  command = the o check_tool "ISABELLE_VERIT",
73388
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   140
  options = veriT_options,
61587
c3974cd2d381 updating options to verit
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 60201
diff changeset
   141
  smt_options = [(":produce-proofs", "true")],
75029
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
   142
  good_slices =
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
   143
    (* FUDGE *)
75339
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   144
    [((1, 1024, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   145
     ((1, 512, mashN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   146
     ((1, 64, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   147
     ((1, 128, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   148
     ((1, 256, mepoN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   149
     ((1, 32, meshN), [])],
74691
634e2323b6cf proper support of verit's return code for timeout
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74553
diff changeset
   150
  outcome = on_first_non_unsupported_line (outcome_of "unsat" "sat" "unknown" "Time limit exceeded"),
75299
da591621d6ae split veriT reconstruction into Lethe and veriT part
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 75063
diff changeset
   151
  parse_proof = SOME (K Lethe_Proof_Parse.parse_proof),
69205
8050734eee3e add reconstruction by veriT in method smt
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 67522
diff changeset
   152
  replay = SOME Verit_Replay.replay }
57240
9a5729600ba9 added support for CVC4 in SMT2
blanchet
parents: 57239
diff changeset
   153
66551
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   154
end
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   155
4df6b0ae900d towards support for HO SMT-LIB
blanchet
parents: 64461
diff changeset
   156
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   157
(* Z3 *)
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   158
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 69205
diff changeset
   159
val z3_extensions = Attrib.setup_config_bool \<^binding>\<open>z3_extensions\<close> (K false)
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   160
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   161
local
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   162
  fun z3_options ctxt =
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   163
    ["smt.random_seed=" ^ string_of_int (Config.get ctxt SMT_Config.random_seed),
73388
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   164
     "smt.refine_inj_axioms=false"] @
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   165
    (case SMT_Config.get_timeout ctxt of
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   166
      NONE => []
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   167
    | SOME t => ["-T:" ^ string_of_int (Real.ceil (Time.toReal t))]) @
a40e69fde2b4 clarified smt: support Timeout.ignored and Timeout.scale_time;
wenzelm
parents: 73104
diff changeset
   168
    ["-smt2"]
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   169
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   170
  fun select_class ctxt =
74817
1fd8705503b4 generate problems with correct logic for veriT
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74691
diff changeset
   171
    if Config.get ctxt z3_extensions then Z3_Interface.smtlib_z3C
1fd8705503b4 generate problems with correct logic for veriT
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74691
diff changeset
   172
    else if Config.get ctxt SMT_Config.native_bv then SMTLIB_Interface.bvsmlibC
1fd8705503b4 generate problems with correct logic for veriT
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 74691
diff changeset
   173
    else SMTLIB_Interface.smtlibC
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   174
in
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   175
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   176
val z3: SMT_Solver.solver_config = {
57209
7ffa0f7e2775 removed '_new' sufffix in SMT2 solver names (in some cases)
blanchet
parents: 57168
diff changeset
   177
  name = "z3",
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   178
  class = select_class,
59960
372ddff01244 updated SMT module and Sledgehammer to fully open source Z3
blanchet
parents: 59035
diff changeset
   179
  avail = make_avail "Z3",
372ddff01244 updated SMT module and Sledgehammer to fully open source Z3
blanchet
parents: 59035
diff changeset
   180
  command = make_command "Z3",
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   181
  options = z3_options,
57239
a40edeaa01b1 don't ask proof-disabled solvers to do proofs
blanchet
parents: 57237
diff changeset
   182
  smt_options = [(":produce-proofs", "true")],
75029
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
   183
  good_slices =
dc6769b86fd6 crude implementation of centralized slicing
blanchet
parents: 74817
diff changeset
   184
    (* FUDGE *)
75339
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   185
    [((1, 1024, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   186
     ((1, 512, mepoN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   187
     ((1, 64, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   188
     ((1, 256, meshN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   189
     ((1, 128, mashN), []),
d9bb81999d2c first step in making time slicing more flexible in Sledgehammer: label slices with 'slice size'
blanchet
parents: 75299
diff changeset
   190
     ((1, 32, meshN), [])],
70327
c04d4951a155 handle timeouts gracefully in 'smt' proof method (patch due to Mathias Fleury)
blanchet
parents: 69593
diff changeset
   191
  outcome = on_first_line (outcome_of "unsat" "sat" "unknown" "timeout"),
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   192
  parse_proof = SOME Z3_Replay.parse_proof,
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   193
  replay = SOME Z3_Replay.replay }
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   194
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   195
end
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   196
72458
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   197
(* smt tactic *)
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   198
val parse_smt_options =
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   199
  Scan.optional
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   200
    (Args.parens (Args.name -- Scan.option (\<^keyword>\<open>,\<close> |-- Args.name)) >> apfst SOME)
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   201
    (NONE, NONE)
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   202
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   203
fun smt_method ((solver, stgy), thms) ctxt facts =
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   204
  let
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   205
    val default_solver = SMT_Config.solver_of ctxt
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   206
    val solver = the_default default_solver solver
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   207
    val _ = 
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   208
      if solver = "z3" andalso stgy <> NONE
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   209
      then warning ("No strategy is available for z3. Ignoring " ^ quote (the stgy)) 
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   210
      else ()
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   211
    val ctxt =
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   212
      ctxt
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   213
      |> (if stgy <> NONE then Context.proof_map (Verit_Proof.select_veriT_stgy (the stgy)) else I)
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   214
      |> Context.Proof
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   215
      |> SMT_Config.select_solver solver
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   216
      |> Context.proof_of
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   217
  in
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   218
    HEADGOAL (SOLVED' (SMT_Solver.smt_tac ctxt (thms @ facts)))
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   219
  end
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   220
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   221
val _ =
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   222
  Theory.setup
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   223
    (Method.setup \<^binding>\<open>smt\<close>
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   224
      (Scan.lift parse_smt_options -- Attrib.thms >> (METHOD oo smt_method))
b44e894796d5 add reconstruction for the SMT solver veriT
Mathias Fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 70327
diff changeset
   225
      "Call to the SMT solvers veriT or z3")
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   226
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   227
(* overall setup *)
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   228
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   229
val _ = Theory.setup (
58061
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   230
  SMT_Solver.add_solver cvc4 #>
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   231
  SMT_Solver.add_solver veriT #>
3d060f43accb renamed new SMT module from 'SMT2' to 'SMT'
blanchet
parents: 57714
diff changeset
   232
  SMT_Solver.add_solver z3)
56078
624faeda77b5 moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
blanchet
parents:
diff changeset
   233
57229
blanchet
parents: 57210
diff changeset
   234
end;