src/Pure/Isar/locale.ML
changeset 17257 0ab67cb765da
parent 17228 19b460b39dad
child 17271 2756a73f63a5
--- a/src/Pure/Isar/locale.ML	Sat Sep 03 22:27:06 2005 +0200
+++ b/src/Pure/Isar/locale.ML	Mon Sep 05 08:14:35 2005 +0200
@@ -1896,10 +1896,10 @@
       Tactic.compose_tac (false, Drule.conj_intr_list (map (Thm.assume o cert) norm_ts), 0) 1));
 
     val conjuncts =
-      Drule.equal_elim_rule1 OF [Thm.symmetric body_eq,
-        Tactic.rewrite_rule [pred_def] (Thm.assume (cert statement))]
+      (Drule.equal_elim_rule1 OF [Thm.symmetric body_eq,
+        Tactic.rewrite_rule [pred_def] (Thm.assume (cert statement))])
       |> Drule.conj_elim_precise (length ts);
-    val axioms = (ts ~~ conjuncts) |> map (fn (t, ax) =>
+    val axioms = ts ~~ conjuncts |> map (fn (t, ax) =>
       Tactic.prove_plain defs_thy [] [] t (fn _ =>
         Tactic.rewrite_goals_tac defs THEN
         Tactic.compose_tac (false, ax, 0) 1));