removed obsolete old goal command;
authorwenzelm
Sat, 17 Oct 2009 01:05:59 +0200
changeset 32959 23a8c5ac35f8
parent 32958 3228627994d9
child 32960 69916a850301
removed obsolete old goal command;
src/HOL/Tools/TFL/post.ML
--- a/src/HOL/Tools/TFL/post.ML	Sat Oct 17 00:53:18 2009 +0200
+++ b/src/HOL/Tools/TFL/post.ML	Sat Oct 17 01:05:59 2009 +0200
@@ -7,8 +7,6 @@
 
 signature TFL =
 sig
-  val tgoalw: theory -> thm list -> thm list -> thm list
-  val tgoal: theory -> thm list -> thm list
   val define_i: bool -> theory -> claset -> simpset -> thm list -> thm list -> xstring ->
     term -> term list -> theory * {rules: (thm * int) list, induct: thm, tcs: term list}
   val define: bool -> theory -> claset -> simpset -> thm list -> thm list -> xstring ->
@@ -33,19 +31,6 @@
       (List.foldr (fn (th,A) => gen_union (op aconv) (prems_of th, A)) [] rules);
 
 (*---------------------------------------------------------------------------
- * Finds the termination conditions in (highly massaged) definition and
- * puts them into a goalstack.
- *--------------------------------------------------------------------------*)
-fun tgoalw thy defs rules =
-  case termination_goals rules of
-      [] => error "tgoalw: no termination conditions to prove"
-    | L  => OldGoals.goalw_cterm defs
-              (Thm.cterm_of thy
-                        (HOLogic.mk_Trueprop(USyntax.list_mk_conj L)));
-
-fun tgoal thy = tgoalw thy [];
-
-(*---------------------------------------------------------------------------
  * Three postprocessors are applied to the definition.  It
  * attempts to prove wellfoundedness of the given relation, simplifies the
  * non-proved termination conditions, and finally attempts to prove the