src/ZF/pair.ML
changeset 3840 e0baea4d485a
parent 2877 6476784dba1c
child 4091 771b1f6422a8
--- a/src/ZF/pair.ML	Fri Oct 10 18:17:17 1997 +0200
+++ b/src/ZF/pair.ML	Fri Oct 10 18:23:31 1997 +0200
@@ -131,7 +131,7 @@
 (*** Eliminator - split ***)
 
 (*A META-equality, so that it applies to higher types as well...*)
-qed_goalw "split" ZF.thy [split_def] "split(%x y.c(x,y), <a,b>) == c(a,b)"
+qed_goalw "split" ZF.thy [split_def] "split(%x y. c(x,y), <a,b>) == c(a,b)"
  (fn _ => [ (Simp_tac 1),
             (rtac reflexive_thm 1) ]);
 
@@ -140,7 +140,7 @@
 qed_goal "split_type" ZF.thy
     "[|  p:Sigma(A,B);   \
 \        !!x y.[| x:A; y:B(x) |] ==> c(x,y):C(<x,y>) \
-\    |] ==> split(%x y.c(x,y), p) : C(p)"
+\    |] ==> split(%x y. c(x,y), p) : C(p)"
  (fn major::prems=>
   [ (rtac (major RS SigmaE) 1),
     (asm_simp_tac (!simpset addsimps prems) 1) ]);