src/Pure/Isar/local_theory.ML
changeset 57941 57200bdc2aa7
parent 57938 a9fa81e150c9
child 58011 bc6bced136e5
--- a/src/Pure/Isar/local_theory.ML	Thu Aug 14 12:49:49 2014 +0200
+++ b/src/Pure/Isar/local_theory.ML	Thu Aug 14 14:28:11 2014 +0200
@@ -39,7 +39,6 @@
   val raw_theory: (theory -> theory) -> local_theory -> local_theory
   val background_theory_result: (theory -> 'a * theory) -> local_theory -> 'a * local_theory
   val background_theory: (theory -> theory) -> local_theory -> local_theory
-  val background_morphism: local_theory -> morphism
   val target_of: local_theory -> Proof.context
   val target: (Proof.context -> Proof.context) -> local_theory -> local_theory
   val target_morphism: local_theory -> morphism
@@ -106,7 +105,8 @@
   target: Proof.context};
 
 fun make_lthy (naming, operations, after_close, brittle, target) : lthy =
-  {naming = naming, operations = operations, after_close = after_close, brittle = brittle, target = target};
+  {naming = naming, operations = operations, after_close = after_close,
+    brittle = brittle, target = target};
 
 
 (* context data *)
@@ -226,9 +226,6 @@
 
 fun background_theory f = #2 o background_theory_result (f #> pair ());
 
-fun background_morphism lthy =
-  standard_morphism lthy (Proof_Context.init_global (Proof_Context.theory_of lthy));
-
 
 (* target contexts *)