src/HOL/ATP_Linkup.thy
author wenzelm
Wed, 21 Jan 2009 20:05:31 +0100
changeset 29600 0182b65e4ad0
parent 29593 7b73bd578db2
parent 29580 117b88da143c
child 29611 9891e3646809
permissions -rw-r--r--
merged
     1 (*  Title:      HOL/ATP_Linkup.thy
     2     Author:     Lawrence C Paulson
     3     Author:     Jia Meng, NICTA
     4     Author:     Fabian Immler, TUM
     5 *)
     6 
     7 header {* The Isabelle-ATP Linkup *}
     8 
     9 theory ATP_Linkup
    10 imports Record Hilbert_Choice
    11 uses
    12   "Tools/polyhash.ML"
    13   "Tools/res_clause.ML"
    14   ("Tools/res_axioms.ML")
    15   ("Tools/res_hol_clause.ML")
    16   ("Tools/res_reconstruct.ML")
    17   ("Tools/res_atp.ML")
    18   ("Tools/atp_manager.ML")
    19   ("Tools/atp_wrapper.ML")
    20   "~~/src/Tools/Metis/metis.ML"
    21   ("Tools/metis_tools.ML")
    22 begin
    23 
    24 definition COMBI :: "'a => 'a"
    25   where "COMBI P == P"
    26 
    27 definition COMBK :: "'a => 'b => 'a"
    28   where "COMBK P Q == P"
    29 
    30 definition COMBB :: "('b => 'c) => ('a => 'b) => 'a => 'c"
    31   where "COMBB P Q R == P (Q R)"
    32 
    33 definition COMBC :: "('a => 'b => 'c) => 'b => 'a => 'c"
    34   where "COMBC P Q R == P R Q"
    35 
    36 definition COMBS :: "('a => 'b => 'c) => ('a => 'b) => 'a => 'c"
    37   where "COMBS P Q R == P R (Q R)"
    38 
    39 definition fequal :: "'a => 'a => bool"
    40   where "fequal X Y == (X=Y)"
    41 
    42 lemma fequal_imp_equal: "fequal X Y ==> X=Y"
    43   by (simp add: fequal_def)
    44 
    45 lemma equal_imp_fequal: "X=Y ==> fequal X Y"
    46   by (simp add: fequal_def)
    47 
    48 text{*These two represent the equivalence between Boolean equality and iff.
    49 They can't be converted to clauses automatically, as the iff would be
    50 expanded...*}
    51 
    52 lemma iff_positive: "P | Q | P=Q"
    53 by blast
    54 
    55 lemma iff_negative: "~P | ~Q | P=Q"
    56 by blast
    57 
    58 text{*Theorems for translation to combinators*}
    59 
    60 lemma abs_S: "(%x. (f x) (g x)) == COMBS f g"
    61 apply (rule eq_reflection)
    62 apply (rule ext) 
    63 apply (simp add: COMBS_def) 
    64 done
    65 
    66 lemma abs_I: "(%x. x) == COMBI"
    67 apply (rule eq_reflection)
    68 apply (rule ext) 
    69 apply (simp add: COMBI_def) 
    70 done
    71 
    72 lemma abs_K: "(%x. y) == COMBK y"
    73 apply (rule eq_reflection)
    74 apply (rule ext) 
    75 apply (simp add: COMBK_def) 
    76 done
    77 
    78 lemma abs_B: "(%x. a (g x)) == COMBB a g"
    79 apply (rule eq_reflection)
    80 apply (rule ext) 
    81 apply (simp add: COMBB_def) 
    82 done
    83 
    84 lemma abs_C: "(%x. (f x) b) == COMBC f b"
    85 apply (rule eq_reflection)
    86 apply (rule ext) 
    87 apply (simp add: COMBC_def) 
    88 done
    89 
    90 
    91 subsection {* Setup of external ATPs *}
    92 
    93 use "Tools/res_axioms.ML" setup ResAxioms.setup
    94 use "Tools/res_hol_clause.ML"
    95 use "Tools/res_reconstruct.ML" setup ResReconstruct.setup
    96 use "Tools/res_atp.ML"
    97 
    98 use "Tools/atp_manager.ML"
    99 use "Tools/atp_wrapper.ML"
   100 
   101 text {* basic provers *}
   102 setup {* AtpManager.add_prover "spass" AtpWrapper.spass *}
   103 setup {* AtpManager.add_prover "vampire" AtpWrapper.vampire *}
   104 setup {* AtpManager.add_prover "e" AtpWrapper.eprover *}
   105 
   106 text {* provers with stuctured output *}
   107 setup {* AtpManager.add_prover "vampire_full" AtpWrapper.vampire_full *}
   108 setup {* AtpManager.add_prover "e_full" AtpWrapper.eprover_full *}
   109 
   110 text {* on some problems better results *}
   111 setup {* AtpManager.add_prover "spass_no_tc" (AtpWrapper.spass_opts 40 false) *}
   112 
   113 text {* remote provers via SystemOnTPTP *}
   114 setup {* AtpManager.add_prover "remote_vampire"
   115   (AtpWrapper.remote_prover "-s Vampire---9.0") *}
   116 setup {* AtpManager.add_prover "remote_spass"
   117   (AtpWrapper.remote_prover "-s SPASS---3.01") *}
   118 setup {* AtpManager.add_prover "remote_e"
   119   (AtpWrapper.remote_prover "-s EP---1.0") *}
   120   
   121 
   122 
   123 subsection {* The Metis prover *}
   124 
   125 use "Tools/metis_tools.ML"
   126 setup MetisTools.setup
   127 
   128 end