src/HOL/SMT/Z3.thy
changeset 33010 39f73a59e855
child 33021 c065b9300d44
equal deleted inserted replaced
33008:b0ff69f0a248 33010:39f73a59e855
       
     1 (*  Title:      HOL/SMT/Z3.thy
       
     2     Author:     Sascha Boehme, TU Muenchen
       
     3 *)
       
     4 
       
     5 header {* Binding to the SMT solver Z3, with proof reconstruction *}
       
     6 
       
     7 theory Z3
       
     8 imports SMT_Base
       
     9 uses
       
    10   "Tools/z3_proof_terms.ML"
       
    11   "Tools/z3_proof_rules.ML"
       
    12   "Tools/z3_proof.ML"
       
    13   "Tools/z3_model.ML"
       
    14   "Tools/z3_interface.ML"
       
    15   "Tools/z3_solver.ML"
       
    16 begin
       
    17 
       
    18 setup {* Z3_Proof_Rules.setup #> Z3_Solver.setup *}
       
    19 
       
    20 lemmas [z3_rewrite] =
       
    21   refl eq_commute conj_commute disj_commute simp_thms nnf_simps
       
    22   ring_distribs field_eq_simps
       
    23 
       
    24 end