src/HOL/Tools/Quotient/quotient_def.ML
changeset 54742 7a86358a3c0b
parent 50902 cb2b940e2fdf
child 55945 e96383acecf9
--- a/src/HOL/Tools/Quotient/quotient_def.ML	Fri Dec 13 23:53:02 2013 +0100
+++ b/src/HOL/Tools/Quotient/quotient_def.ML	Sat Dec 14 17:28:05 2013 +0100
@@ -129,7 +129,7 @@
     val eq_thm = 
       (simp_conv then_conv univq_prenex_conv then_conv beta_conv then_conv unfold_ret_val_invs) ctm
   in
-    Object_Logic.rulify (eq_thm RS Drule.equal_elim_rule2)
+    Object_Logic.rulify lthy (eq_thm RS Drule.equal_elim_rule2)
   end
 
 
@@ -187,7 +187,7 @@
           case thm_list of
             [] => the maybe_proven_rsp_thm
           | [[thm]] => Goal.prove ctxt [] [] internal_rsp_tm 
-            (fn _ => rtac readable_rsp_thm_eq 1 THEN Proof_Context.fact_tac [thm] 1)
+            (fn _ => rtac readable_rsp_thm_eq 1 THEN Proof_Context.fact_tac ctxt [thm] 1)
       in
         snd (add_quotient_def ((var, attr), (lhs, rhs)) internal_rsp_thm lthy)
       end