src/HOL/Tools/Ctr_Sugar/ctr_sugar.ML
changeset 59621 291934bac95e
parent 59582 0fbed69ff081
child 59647 c6f413b660cf
--- a/src/HOL/Tools/Ctr_Sugar/ctr_sugar.ML	Fri Mar 06 14:01:08 2015 +0100
+++ b/src/HOL/Tools/Ctr_Sugar/ctr_sugar.ML	Fri Mar 06 15:58:56 2015 +0100
@@ -679,10 +679,10 @@
       let
         val ((inject_thms, inject_thmss), half_distinct_thmss) = chop n thmss |>> `flat;
 
-        val rho_As = map (apply2 (Proof_Context.ctyp_of lthy)) (map Logic.varifyT_global As ~~ As);
+        val rho_As = map (apply2 (Thm.ctyp_of lthy)) (map Logic.varifyT_global As ~~ As);
 
         fun inst_thm t thm =
-          Drule.instantiate' [] [SOME (Proof_Context.cterm_of lthy t)]
+          Drule.instantiate' [] [SOME (Thm.cterm_of lthy t)]
             (Thm.instantiate (rho_As, []) (Drule.zero_var_indexes thm));
 
         val uexhaust_thm = inst_thm u exhaust_thm;
@@ -997,7 +997,7 @@
                     mk_Trueprop_eq (udisc, list_comb (casexBool, mk_case_args n) $ u)) udiscs;
                 in
                   Goal.prove_sorry lthy [] [] (Logic.mk_conjunction_balanced goals)
-                    (fn {context = ctxt, ...} => mk_disc_eq_case_tac ctxt (Proof_Context.cterm_of ctxt u)
+                    (fn {context = ctxt, ...} => mk_disc_eq_case_tac ctxt (Thm.cterm_of ctxt u)
                        exhaust_thm (flat nontriv_disc_thmss) distinct_thms case_thms)
                   |> Conjunction.elim_balanced (length goals)
                   |> Proof_Context.export names_lthy lthy
@@ -1020,7 +1020,7 @@
             val goal = mk_Trueprop_eq (h $ ufcase, list_comb (casexC, args) $ u);
           in
             Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, ...} =>
-              mk_case_distrib_tac ctxt (Proof_Context.cterm_of ctxt u) exhaust_thm case_thms)
+              mk_case_distrib_tac ctxt (Thm.cterm_of ctxt u) exhaust_thm case_thms)
             |> singleton (Proof_Context.export names_lthy lthy)
             |> Thm.close_derivation
           end;