TFL/thms.ML
author wenzelm
Fri, 26 Oct 2001 23:58:21 +0200
changeset 11952 b10f1e8862f4
parent 11455 e07927b980ec
permissions -rw-r--r--
* Pure: method 'atomize' presents local goal premises as object-level statements (atomic meta-level propositions); setup controlled via rewrite rules declarations of 'atomize' attribute; example application: 'induct' method with proper rule statements in improper proof *scripts*;

(*  Title:      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;