src/HOL/Metis.thy
changeset 43085 0a2f5b86bdd7
parent 43016 42330f25142c
child 44651 5d6a11e166cf
--- a/src/HOL/Metis.thy	Tue May 31 11:21:47 2011 +0200
+++ b/src/HOL/Metis.thy	Tue May 31 16:38:36 2011 +0200
@@ -7,7 +7,7 @@
 header {* Metis Proof Method *}
 
 theory Metis
-imports Meson
+imports ATP
 uses "~~/src/Tools/Metis/metis.ML"
      ("Tools/Metis/metis_translate.ML")
      ("Tools/Metis/metis_reconstruct.ML")
@@ -15,31 +15,6 @@
      ("Tools/try_methods.ML")
 begin
 
-
-subsection {* Higher-order reasoning helpers *}
-
-definition fFalse :: bool where [no_atp]:
-"fFalse \<longleftrightarrow> False"
-
-definition fTrue :: bool where [no_atp]:
-"fTrue \<longleftrightarrow> True"
-
-definition fNot :: "bool \<Rightarrow> bool" where [no_atp]:
-"fNot P \<longleftrightarrow> \<not> P"
-
-definition fconj :: "bool \<Rightarrow> bool \<Rightarrow> bool" where [no_atp]:
-"fconj P Q \<longleftrightarrow> P \<and> Q"
-
-definition fdisj :: "bool \<Rightarrow> bool \<Rightarrow> bool" where [no_atp]:
-"fdisj P Q \<longleftrightarrow> P \<or> Q"
-
-definition fimplies :: "bool \<Rightarrow> bool \<Rightarrow> bool" where [no_atp]:
-"fimplies P Q \<longleftrightarrow> (P \<longrightarrow> Q)"
-
-definition fequal :: "'a \<Rightarrow> 'a \<Rightarrow> bool" where [no_atp]:
-"fequal x y \<longleftrightarrow> (x = y)"
-
-
 subsection {* Literal selection helpers *}
 
 definition select :: "'a \<Rightarrow> 'a" where