src/HOL/Tools/Predicate_Compile/code_prolog.ML
changeset 52788 da1fdbfebd39
parent 51709 19b47bfac6ef
child 55399 5c8e91f884af
child 55437 3fd63b92ea3b
--- a/src/HOL/Tools/Predicate_Compile/code_prolog.ML	Tue Jul 30 12:07:14 2013 +0200
+++ b/src/HOL/Tools/Predicate_Compile/code_prolog.ML	Tue Jul 30 15:09:25 2013 +0200
@@ -941,7 +941,7 @@
     val T = Sign.the_const_type (Proof_Context.theory_of ctxt) name
     val t = Const (name, T)
     val thy' =
-      Theory.copy (Proof_Context.theory_of ctxt)
+      Proof_Context.theory_of ctxt
       |> Predicate_Compile.preprocess preprocess_options t
     val ctxt' = Proof_Context.init_global thy'
     val _ = tracing "Generating prolog program..."
@@ -1020,7 +1020,7 @@
   let
     val t' = fold_rev absfree (Term.add_frees t []) t
     val options = code_options_of (Proof_Context.theory_of ctxt)
-    val thy = Theory.copy (Proof_Context.theory_of ctxt)
+    val thy = Proof_Context.theory_of ctxt
     val ((((full_constname, constT), vs'), intro), thy1) =
       Predicate_Compile_Aux.define_quickcheck_predicate t' thy
     val thy2 = Context.theory_map (Predicate_Compile_Alternative_Defs.add_thm intro) thy1