src/HOL/Tools/datatype_realizer.ML
changeset 18358 0a733e11021a
parent 17959 8db36a108213
child 18929 d81435108688
--- a/src/HOL/Tools/datatype_realizer.ML	Tue Dec 06 06:22:14 2005 +0100
+++ b/src/HOL/Tools/datatype_realizer.ML	Tue Dec 06 09:04:09 2005 +0100
@@ -130,11 +130,11 @@
 
     val ind_name = Thm.name_of_thm induction;
     val vs = map (fn i => List.nth (pnames, i)) is;
-    val (thy', thm') = thy
+    val (thm', thy') = thy
       |> Theory.absolute_path
       |> PureThy.store_thm
         ((space_implode "_" (ind_name :: vs @ ["correctness"]), thm), [])
-      |>> Theory.restore_naming thy;
+      ||> Theory.restore_naming thy;
 
     val ivs = Drule.vars_of_terms
       [Logic.varify (DatatypeProp.make_ind [descr] sorts)];
@@ -200,10 +200,10 @@
              resolve_tac prems, asm_simp_tac HOL_basic_ss])]);
 
     val exh_name = Thm.name_of_thm exhaustion;
-    val (thy', thm') = thy
+    val (thm', thy') = thy
       |> Theory.absolute_path
       |> PureThy.store_thm ((exh_name ^ "_P_correctness", thm), [])
-      |>> Theory.restore_naming thy;
+      ||> Theory.restore_naming thy;
 
     val P = Var (("P", 0), rT' --> HOLogic.boolT);
     val prf = forall_intr_prf (y, forall_intr_prf (P,