TFL/rules.ML
changeset 17892 62c397c17d18
parent 17203 29b2563f5c11
child 17959 8db36a108213
--- a/TFL/rules.ML	Tue Oct 18 17:59:24 2005 +0200
+++ b/TFL/rules.ML	Tue Oct 18 17:59:25 2005 +0200
@@ -664,7 +664,8 @@
 
 fun CONTEXT_REWRITE_RULE (func, G, cut_lemma, congs) th =
  let val globals = func::G
-     val pbeta_reduce = simpl_conv empty_ss [split_conv RS eq_reflection];
+     val ss0 = Simplifier.theory_context (Thm.theory_of_thm th) empty_ss
+     val pbeta_reduce = simpl_conv ss0 [split_conv RS eq_reflection];
      val tc_list = ref[]: term list ref
      val dummy = term_ref := []
      val dummy = thm_ref  := []
@@ -805,7 +806,7 @@
     val ctm = cprop_of th
     val names = add_term_names (term_of ctm, [])
     val th1 = MetaSimplifier.rewrite_cterm(false,true,false)
-      (prover names) (empty_ss addsimps [cut_lemma'] addeqcongs congs) ctm
+      (prover names) (ss0 addsimps [cut_lemma'] addeqcongs congs) ctm
     val th2 = equal_elim th1 th
  in
  (th2, List.filter (not o restricted) (!tc_list))