removed export_thm;
authorwenzelm
Tue, 23 Oct 2001 19:15:00 +0200
changeset 11906 a71713885e3e
parent 11905 77c63f8e9d9a
child 11907 f2a5481c7998
removed export_thm;
src/Pure/Isar/proof.ML
--- a/src/Pure/Isar/proof.ML	Tue Oct 23 19:14:47 2001 +0200
+++ b/src/Pure/Isar/proof.ML	Tue Oct 23 19:15:00 2001 +0200
@@ -50,7 +50,6 @@
   val method_cases: (thm list -> thm -> (thm * (string * RuleCases.T) list) Seq.seq) -> method
   val refine: (context -> method) -> state -> state Seq.seq
   val refine_end: (context -> method) -> state -> state Seq.seq
-  val export_thm: context -> thm -> thm
   val match_bind: (string list * string) list -> state -> state
   val match_bind_i: (term list * term) list -> state -> state
   val let_bind: (string list * string) list -> state -> state
@@ -430,14 +429,6 @@
       in Seq.map (fn th => map_goal I (K ((result, (facts, th)), f)) state) thmq end;
   in raw_rule |> exp_tac |> (Seq.flat o Seq.map exp_rule) end;
 
-fun export_thm inner thm =
-  let val exp_tac = ProofContext.export_wrt false inner None in
-    (case Seq.chop (2, exp_tac thm) of
-      ([thm'], _) => thm'
-    | ([], _) => raise THM ("export: failed", 0, [thm])
-    | _ => raise THM ("export: more than one result", 0, [thm]))
-  end;
-
 fun transfer_facts inner_state state =
   (case get_facts inner_state of
     None => Seq.single (reset_facts state)