src/ZF/pair.ML
changeset 6112 5e4871c5136b
parent 5505 b0856ff6fc69
child 6153 bff90585cce5
--- a/src/ZF/pair.ML	Wed Jan 13 11:56:28 1999 +0100
+++ b/src/ZF/pair.ML	Wed Jan 13 11:57:09 1999 +0100
@@ -135,10 +135,9 @@
 (*** Eliminator - split ***)
 
 (*A META-equality, so that it applies to higher types as well...*)
-qed_goalw "split" thy [split_def] "split(%x y. c(x,y), <a,b>) == c(a,b)"
- (fn _ => [ (Simp_tac 1),
-            (rtac reflexive_thm 1) ]);
-
+Goalw [split_def] "split(%x y. c(x,y), <a,b>) == c(a,b)";
+by (Simp_tac 1);
+qed "split";
 Addsimps [split];
 
 qed_goal "split_type" thy