src/Tools/more_conv.ML
changeset 32843 c8f5a7c8353f
parent 32821 99843bbfaeb2
--- a/src/Tools/more_conv.ML	Thu Oct 01 22:40:29 2009 +0200
+++ b/src/Tools/more_conv.ML	Thu Oct 01 23:27:05 2009 +0200
@@ -1,5 +1,5 @@
-(* Title:  Tools/more_conv.ML
-   Author: Sascha Boehme
+(*  Title:       Tools/more_conv.ML
+    Author:      Sascha Boehme, TU Muenchen
 
 Further conversions and conversionals.
 *)
@@ -14,16 +14,11 @@
   val top_sweep_conv: (Proof.context -> conv) -> Proof.context -> conv
 
   val binder_conv: (Proof.context -> conv) -> Proof.context -> conv
-
-  val cache_conv: conv -> conv
 end
 
-
-
 structure More_Conv : MORE_CONV =
 struct
 
-
 fun rewrs_conv eqs = Conv.first_conv (map Conv.rewr_conv eqs)
 
 
@@ -45,19 +40,4 @@
 fun binder_conv cv ctxt =
   Conv.arg_conv (Conv.abs_conv (fn (_, cx) => cv cx) ctxt)
 
-
-fun cache_conv conv =
-  let
-    val cache = Synchronized.var "cache_conv" Termtab.empty
-    fun lookup t =
-      Synchronized.change_result cache (fn tab => (Termtab.lookup tab t, tab))
-    val keep = Synchronized.change cache o Termtab.insert Thm.eq_thm
-    fun keep_result t thm = (keep (t, thm); thm)
-
-    fun cconv ct =
-      (case lookup (Thm.term_of ct) of
-        SOME thm => thm
-      | NONE => keep_result (Thm.term_of ct) (conv ct))
-  in cconv end
-
 end