src/ZF/pair.ML
changeset 6153 bff90585cce5
parent 6112 5e4871c5136b
child 9180 3bda56c0d70d
--- a/src/ZF/pair.ML	Mon Jan 25 20:35:19 1999 +0100
+++ b/src/ZF/pair.ML	Wed Jan 27 10:31:31 1999 +0100
@@ -63,6 +63,7 @@
 qed_goal "SigmaI" thy
     "!!a b. [| a:A;  b:B(a) |] ==> <a,b> : Sigma(A,B)"
  (fn _ => [ Asm_simp_tac 1 ]);
+AddTCs [SigmaI];
 
 bind_thm ("SigmaD1", Sigma_iff RS iffD1 RS conjunct1);
 bind_thm ("SigmaD2", Sigma_iff RS iffD1 RS conjunct2);
@@ -147,6 +148,7 @@
  (fn major::prems=>
   [ (rtac (major RS SigmaE) 1),
     (asm_simp_tac (simpset() addsimps prems) 1) ]);
+AddTCs [split_type];
 
 Goalw [split_def]
   "u: A*B ==>   \