removed obsolete Proof.get_thmss_cmd (cf. Attrib.eval_thms);
authorwenzelm
Wed, 11 Aug 2010 17:37:04 +0200
changeset 38333 3f4fadad9497
parent 38332 6551e310e7cb
child 38334 c677c2c1d333
removed obsolete Proof.get_thmss_cmd (cf. Attrib.eval_thms);
src/Pure/Isar/proof.ML
--- a/src/Pure/Isar/proof.ML	Wed Aug 11 17:31:56 2010 +0200
+++ b/src/Pure/Isar/proof.ML	Wed Aug 11 17:37:04 2010 +0200
@@ -60,7 +60,6 @@
   val def_cmd: (Attrib.binding * ((binding * mixfix) * (string * string list))) list -> state -> state
   val chain: state -> state
   val chain_facts: thm list -> state -> state
-  val get_thmss_cmd: state -> (Facts.ref * Attrib.src list) list -> thm list
   val note_thmss: (Thm.binding * (thm list * attribute list) list) list -> state -> state
   val note_thmss_cmd: (Attrib.binding * (Facts.ref * Attrib.src list) list) list -> state -> state
   val from_thmss: ((thm list * attribute list) list) list -> state -> state
@@ -679,8 +678,6 @@
 
 val local_results = gen_thmss (K []) I I (K I) (K I) o map (apsnd Thm.simple_fact);
 
-fun get_thmss_cmd state srcs = the_facts (note_thmss_cmd [((Binding.empty, []), srcs)] state);
-
 end;