proper Proof_Context.export_morphism corresponding to Proof_Context.augment (see 7f568724d67e);
authorwenzelm
Tue, 04 Jun 2019 15:11:29 +0200
changeset 70318 9eff9e2dc177
parent 70317 9fced5690f4e
child 70319 34bc296374ee
proper Proof_Context.export_morphism corresponding to Proof_Context.augment (see 7f568724d67e);
src/HOL/Tools/Function/fun_cases.ML
src/HOL/Tools/inductive.ML
--- a/src/HOL/Tools/Function/fun_cases.ML	Tue Jun 04 13:44:59 2019 +0200
+++ b/src/HOL/Tools/Function/fun_cases.ML	Tue Jun 04 15:11:29 2019 +0200
@@ -33,7 +33,7 @@
     fun mk_elim rl =
       Thm.implies_intr cprop
         (Tactic.rule_by_tactic ctxt (Inductive.mk_cases_tac ctxt) (Thm.assume cprop RS rl))
-      |> singleton (Variable.export (Proof_Context.augment prop ctxt) ctxt);
+      |> singleton (Proof_Context.export (Proof_Context.augment prop ctxt) ctxt);
   in
     (case get_first (try mk_elim) (flat elims) of
       SOME r => r
--- a/src/HOL/Tools/inductive.ML	Tue Jun 04 13:44:59 2019 +0200
+++ b/src/HOL/Tools/inductive.ML	Tue Jun 04 15:11:29 2019 +0200
@@ -594,7 +594,7 @@
     fun mk_elim rl =
       Thm.implies_intr cprop
         (Tactic.rule_by_tactic ctxt (mk_cases_tac ctxt) (Thm.assume cprop RS rl))
-      |> singleton (Variable.export (Proof_Context.augment prop ctxt) ctxt);
+      |> singleton (Proof_Context.export (Proof_Context.augment prop ctxt) ctxt);
   in
     (case get_first (try mk_elim) elims of
       SOME r => r
@@ -661,7 +661,7 @@
   in
     infer_instantiate ctxt' inst eq
     |> Conv.fconv_rule (Conv.arg_conv (Conv.arg_conv (Simplifier.full_rewrite ctxt')))
-    |> singleton (Variable.export ctxt' ctxt)
+    |> singleton (Proof_Context.export ctxt' ctxt)
   end