Moved old inductive package to old_inductive_package.ML
authorberghofe
Fri, 13 Oct 2006 18:28:51 +0200
changeset 21025 10b0821a4d11
parent 21024 63ab84bb64d1
child 21026 3b2821e0d541
Moved old inductive package to old_inductive_package.ML
src/HOL/Tools/function_package/inductive_wrap.ML
src/HOLCF/fixrec_package.ML
--- a/src/HOL/Tools/function_package/inductive_wrap.ML	Fri Oct 13 18:27:27 2006 +0200
+++ b/src/HOL/Tools/function_package/inductive_wrap.ML	Fri Oct 13 18:28:51 2006 +0200
@@ -64,7 +64,7 @@
             val qdefs = map dest_all_all cdefs
 
             val (thy, {intrs = intrs_gen, elims = [elim_gen], ...}) =
-                InductivePackage.add_inductive_i true (*verbose*)
+                OldInductivePackage.add_inductive_i true (*verbose*)
                                                  false (* dont add_consts *)
                                                  "" (* no altname *)
                                                  false (* no coind *)
--- a/src/HOLCF/fixrec_package.ML	Fri Oct 13 18:27:27 2006 +0200
+++ b/src/HOLCF/fixrec_package.ML	Fri Oct 13 18:28:51 2006 +0200
@@ -231,7 +231,7 @@
     val eqn_ts = map (prep_prop thy) strings;
     val rec_ts = map (fn eq => chead_of (fst (dest_eqs (Logic.strip_imp_concl eq)))
       handle TERM _ => fixrec_eq_err thy "not a proper equation" eq) eqn_ts;
-    val (_, eqn_ts') = InductivePackage.unify_consts thy rec_ts eqn_ts;
+    val (_, eqn_ts') = OldInductivePackage.unify_consts thy rec_ts eqn_ts;
     
     fun unconcat [] _ = []
       | unconcat (n::ns) xs = List.take (xs,n) :: unconcat ns (List.drop (xs,n));