src/ZF/Datatype_ZF.thy
changeset 61144 5e94dfead1c2
parent 60770 240563fbf41d
child 62913 13252110a6fe
--- a/src/ZF/Datatype_ZF.thy	Wed Sep 09 14:47:41 2015 +0200
+++ b/src/ZF/Datatype_ZF.thy	Wed Sep 09 20:57:21 2015 +0200
@@ -70,8 +70,9 @@
 
  val datatype_ss = simpset_of @{context};
 
- fun proc ctxt old =
-   let val thy = Proof_Context.theory_of ctxt
+ fun proc ctxt ct =
+   let val old = Thm.term_of ct
+       val thy = Proof_Context.theory_of ctxt
        val _ =
          if !trace then writeln ("data_free: OLD = " ^ Syntax.string_of_term ctxt old)
          else ()
@@ -104,7 +105,9 @@
    handle Match => NONE;
 
 
- val conv = Simplifier.simproc_global @{theory} "data_free" ["(x::i) = y"] proc;
+  val conv =
+    Simplifier.make_simproc @{context} "data_free"
+     {lhss = [@{term "(x::i) = y"}], proc = K proc, identifier = []};
 
 end;
 \<close>