--- a/src/HOL/Sledgehammer.thy Fri Mar 19 06:14:37 2010 +0100
+++ b/src/HOL/Sledgehammer.thy Fri Mar 19 13:02:18 2010 +0100
@@ -1,7 +1,8 @@
(* Title: HOL/Sledgehammer.thy
Author: Lawrence C Paulson
Author: Jia Meng, NICTA
- Author: Fabian Immler, TUM
+ Author: Fabian Immler, TU Muenchen
+ Author: Jasmin Blanchette, TU Muenchen
*)
header {* Sledgehammer: Isabelle--ATP Linkup *}
@@ -10,7 +11,8 @@
imports Plain Hilbert_Choice
uses
"Tools/polyhash.ML"
- "Tools/Sledgehammer/sledgehammer_fol_clause.ML"
+ "~~/src/Tools/Metis/metis.ML"
+ ("Tools/Sledgehammer/sledgehammer_fol_clause.ML")
("Tools/Sledgehammer/sledgehammer_fact_preprocessor.ML")
("Tools/Sledgehammer/sledgehammer_hol_clause.ML")
("Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML")
@@ -18,79 +20,79 @@
("Tools/ATP_Manager/atp_manager.ML")
("Tools/ATP_Manager/atp_wrapper.ML")
("Tools/ATP_Manager/atp_minimal.ML")
- "~~/src/Tools/Metis/metis.ML"
+ ("Tools/Sledgehammer/meson_tactic.ML")
("Tools/Sledgehammer/metis_tactics.ML")
begin
-definition COMBI :: "'a => 'a"
- where "COMBI P == P"
+definition COMBI :: "'a \<Rightarrow> 'a"
+ where "COMBI P \<equiv> P"
-definition COMBK :: "'a => 'b => 'a"
- where "COMBK P Q == P"
+definition COMBK :: "'a \<Rightarrow> 'b \<Rightarrow> 'a"
+ where "COMBK P Q \<equiv> P"
-definition COMBB :: "('b => 'c) => ('a => 'b) => 'a => 'c"
- where "COMBB P Q R == P (Q R)"
+definition COMBB :: "('b => 'c) \<Rightarrow> ('a => 'b) \<Rightarrow> 'a \<Rightarrow> 'c"
+ where "COMBB P Q R \<equiv> P (Q R)"
-definition COMBC :: "('a => 'b => 'c) => 'b => 'a => 'c"
- where "COMBC P Q R == P R Q"
+definition COMBC :: "('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'b \<Rightarrow> 'a \<Rightarrow> 'c"
+ where "COMBC P Q R \<equiv> P R Q"
-definition COMBS :: "('a => 'b => 'c) => ('a => 'b) => 'a => 'c"
- where "COMBS P Q R == P R (Q R)"
+definition COMBS :: "('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> ('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'c"
+ where "COMBS P Q R \<equiv> P R (Q R)"
-definition fequal :: "'a => 'a => bool"
- where "fequal X Y == (X=Y)"
+definition fequal :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
+ where "fequal X Y \<equiv> (X = Y)"
-lemma fequal_imp_equal: "fequal X Y ==> X=Y"
+lemma fequal_imp_equal: "fequal X Y \<Longrightarrow> X = Y"
by (simp add: fequal_def)
-lemma equal_imp_fequal: "X=Y ==> fequal X Y"
+lemma equal_imp_fequal: "X = Y \<Longrightarrow> fequal X Y"
by (simp add: fequal_def)
text{*These two represent the equivalence between Boolean equality and iff.
They can't be converted to clauses automatically, as the iff would be
expanded...*}
-lemma iff_positive: "P | Q | P=Q"
+lemma iff_positive: "P \<or> Q \<or> P = Q"
by blast
-lemma iff_negative: "~P | ~Q | P=Q"
+lemma iff_negative: "\<not> P \<or> \<not> Q \<or> P = Q"
by blast
text{*Theorems for translation to combinators*}
-lemma abs_S: "(%x. (f x) (g x)) == COMBS f g"
+lemma abs_S: "\<lambda>x. (f x) (g x) \<equiv> COMBS f g"
apply (rule eq_reflection)
apply (rule ext)
apply (simp add: COMBS_def)
done
-lemma abs_I: "(%x. x) == COMBI"
+lemma abs_I: "\<lambda>x. x \<equiv> COMBI"
apply (rule eq_reflection)
apply (rule ext)
apply (simp add: COMBI_def)
done
-lemma abs_K: "(%x. y) == COMBK y"
+lemma abs_K: "\<lambda>x. y \<equiv> COMBK y"
apply (rule eq_reflection)
apply (rule ext)
apply (simp add: COMBK_def)
done
-lemma abs_B: "(%x. a (g x)) == COMBB a g"
+lemma abs_B: "\<lambda>x. a (g x) \<equiv> COMBB a g"
apply (rule eq_reflection)
apply (rule ext)
apply (simp add: COMBB_def)
done
-lemma abs_C: "(%x. (f x) b) == COMBC f b"
+lemma abs_C: "\<lambda>x. (f x) b \<equiv> COMBC f b"
apply (rule eq_reflection)
apply (rule ext)
apply (simp add: COMBC_def)
done
-
subsection {* Setup of external ATPs *}
+use "Tools/Sledgehammer/sledgehammer_fol_clause.ML"
use "Tools/Sledgehammer/sledgehammer_fact_preprocessor.ML"
setup Sledgehammer_Fact_Preprocessor.setup
use "Tools/Sledgehammer/sledgehammer_hol_clause.ML"
@@ -119,7 +121,12 @@
setup {* ATP_Manager.add_prover ATP_Wrapper.remote_vampire *}
setup {* ATP_Manager.add_prover ATP_Wrapper.remote_spass *}
setup {* ATP_Manager.add_prover ATP_Wrapper.remote_eprover *}
-
+
+
+subsection {* The MESON prover *}
+
+use "Tools/Sledgehammer/meson_tactic.ML"
+setup Meson_Tactic.setup
subsection {* The Metis prover *}