src/HOL/Tools/TFL/thms.ML
changeset 23150 073a65f0bc40
child 39159 0dec18004e75
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Tools/TFL/thms.ML	Thu May 31 13:18:52 2007 +0200
@@ -0,0 +1,20 @@
+(*  Title:      HOL/Tools/TFL/thms.ML
+    ID:         $Id$
+    Author:     Konrad Slind, Cambridge University Computer Laboratory
+    Copyright   1997  University of Cambridge
+*)
+
+structure Thms =
+struct
+  val WFREC_COROLLARY = thm "tfl_wfrec";
+  val WF_INDUCTION_THM = thm "tfl_wf_induct";
+  val CUT_DEF = thm "cut_def";
+  val eqT = thm "tfl_eq_True";
+  val rev_eq_mp = thm "tfl_rev_eq_mp";
+  val simp_thm = thm "tfl_simp_thm";
+  val P_imp_P_iff_True = thm "tfl_P_imp_P_iff_True";
+  val imp_trans = thm "tfl_imp_trans";
+  val disj_assoc = thm "tfl_disj_assoc";
+  val tfl_disjE = thm "tfl_disjE";
+  val choose_thm = thm "tfl_exE";
+end;