src/HOL/Metis.thy
changeset 39946 78faa9b31202
child 39947 f95834c8bb4d
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Metis.thy	Mon Oct 04 22:45:09 2010 +0200
@@ -0,0 +1,35 @@
+(*  Title:      HOL/Metis.thy
+    Author:     Lawrence C. Paulson, Cambridge University Computer Laboratory
+    Author:     Jia Meng, Cambridge University Computer Laboratory and NICTA
+    Author:     Jasmin Blanchette, TU Muenchen
+*)
+
+header {* Metis Proof Method *}
+
+theory Metis
+imports Meson
+uses "~~/src/Tools/Metis/metis.ML"
+     ("Tools/Metis/metis_translate.ML")
+     ("Tools/Metis/metis_reconstruct.ML")
+     ("Tools/Metis/metis_tactics.ML")
+begin
+
+definition fequal :: "'a \<Rightarrow> 'a \<Rightarrow> bool" where [no_atp]:
+"fequal X Y \<longleftrightarrow> (X = Y)"
+
+lemma fequal_imp_equal [no_atp]: "\<not> fequal X Y \<or> X = Y"
+by (simp add: fequal_def)
+
+lemma equal_imp_fequal [no_atp]: "\<not> X = Y \<or> fequal X Y"
+by (simp add: fequal_def)
+
+lemma equal_imp_equal [no_atp]: "X = Y ==> X = Y"
+by auto
+
+use "Tools/Metis/metis_translate.ML"
+use "Tools/Metis/metis_reconstruct.ML"
+use "Tools/Metis/metis_tactics.ML"
+
+setup Metis_Tactics.setup
+
+end