src/ZF/upair.ML
changeset 6153 bff90585cce5
parent 6068 2d8f3e1f1151
child 6163 be8234f37e48
--- a/src/ZF/upair.ML	Mon Jan 25 20:35:19 1999 +0100
+++ b/src/ZF/upair.ML	Wed Jan 27 10:31:31 1999 +0100
@@ -141,6 +141,8 @@
  (fn _ => [ Simp_tac 1 ]);
 
 Addsimps [consI1];
+AddTCs   [consI1];   (*risky as a typechecking rule, but solves otherwise
+		       unconstrained goals of the form  x : ?A*)
 
 qed_goal "consI2" thy "!!B. a : B ==> a : cons(b,B)"
  (fn _ => [ Asm_simp_tac 1 ]);
@@ -288,7 +290,7 @@
     "[| P ==> a: A;  ~P ==> b: A |] ==> (if P then a else b): A"
  (fn prems=> [ (simp_tac 
                 (simpset() addsimps prems addsplits [split_if]) 1) ]);
-
+AddTCs [if_type];
 
 (*** Foundation lemmas ***)