src/ZF/Tools/inductive_package.ML
changeset 51717 9e7d1c139569
parent 50239 fb579401dc26
child 51798 ad3a241def73
--- a/src/ZF/Tools/inductive_package.ML	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/ZF/Tools/inductive_package.ML	Thu Apr 18 17:07:01 2013 +0200
@@ -269,7 +269,7 @@
     Proposition A should have the form t:Si where Si is an inductive set*)
   fun make_cases ctxt A =
     rule_by_tactic ctxt
-      (basic_elim_tac THEN ALLGOALS (asm_full_simp_tac (simpset_of ctxt)) THEN basic_elim_tac)
+      (basic_elim_tac THEN ALLGOALS (asm_full_simp_tac ctxt) THEN basic_elim_tac)
       (Thm.assume A RS elim)
       |> Drule.export_without_context_open;
 
@@ -330,7 +330,7 @@
            (Simplifier.global_context thy empty_ss
              |> Simplifier.set_mksimps (K (map mk_eq o ZF_atomize o gen_all)))
            setSolver (mk_solver "minimal"
-                      (fn ss => resolve_tac (triv_rls @ Simplifier.prems_of ss)
+                      (fn ctxt => resolve_tac (triv_rls @ Simplifier.prems_of ctxt)
                                    ORELSE' assume_tac
                                    ORELSE' etac @{thm FalseE}));