simplified LocalTheory.reinit;
authorwenzelm
Mon, 05 Nov 2007 20:50:42 +0100
changeset 25289 3d332d8a827c
parent 25288 6e0c8dd213df
child 25290 250c7a0205ca
simplified LocalTheory.reinit;
src/HOL/Tools/function_package/fundef_datatype.ML
src/Pure/Isar/local_theory.ML
src/Pure/Isar/subclass.ML
--- a/src/HOL/Tools/function_package/fundef_datatype.ML	Mon Nov 05 20:50:41 2007 +0100
+++ b/src/HOL/Tools/function_package/fundef_datatype.ML	Mon Nov 05 20:50:42 2007 +0100
@@ -306,7 +306,7 @@
     lthy
       |> FundefPackage.add_fundef fixes statements config flags
       |> by_pat_completeness_simp
-      |> (fn lthy => LocalTheory.reinit lthy (ProofContext.theory_of lthy))
+      |> LocalTheory.reinit
       |> termination_by_lexicographic_order
 
 val _ =
--- a/src/Pure/Isar/local_theory.ML	Mon Nov 05 20:50:41 2007 +0100
+++ b/src/Pure/Isar/local_theory.ML	Mon Nov 05 20:50:42 2007 +0100
@@ -41,7 +41,7 @@
   val target_name: local_theory -> bstring -> string
   val init: string -> operations -> Proof.context -> local_theory
   val restore: local_theory -> local_theory
-  val reinit: local_theory -> theory -> local_theory
+  val reinit: local_theory -> local_theory
   val exit: local_theory -> Proof.context
 end;
 
@@ -67,7 +67,7 @@
   term_syntax: declaration -> local_theory -> local_theory,
   declaration: declaration -> local_theory -> local_theory,
   target_naming: local_theory -> NameSpace.naming,
-  reinit: local_theory -> theory -> local_theory,
+  reinit: local_theory -> local_theory,
   exit: local_theory -> Proof.context};
 
 datatype lthy = LThy of
--- a/src/Pure/Isar/subclass.ML	Mon Nov 05 20:50:41 2007 +0100
+++ b/src/Pure/Isar/subclass.ML	Mon Nov 05 20:50:42 2007 +0100
@@ -38,7 +38,7 @@
       |> map (ObjectLogic.ensure_propT thy);
     fun after_qed thms =
       LocalTheory.theory (Class.prove_subclass (sub, sup) thms ctxt)
-      #> (fn lthy => LocalTheory.reinit lthy (ProofContext.theory_of (LocalTheory.target_of lthy)));
+      #> LocalTheory.reinit;
   in
     do_proof after_qed sublocale_prop lthy
   end;