src/HOL/Product_Type.thy
changeset 42083 e1209fc7ecdc
parent 42059 83f3dc509068
child 42247 12fe41a92cd5
--- a/src/HOL/Product_Type.thy	Thu Mar 24 16:47:24 2011 +0100
+++ b/src/HOL/Product_Type.thy	Thu Mar 24 16:56:19 2011 +0100
@@ -272,7 +272,7 @@
   fun contract Q f ts =
     case ts of
       [A, Abs(_, _, (s as Const (@{const_syntax prod_case},_) $ t) $ Bound 0)]
-      => if loose_bvar1 (t,0) then f ts else Syntax.const Q $ A $ s
+      => if Term.is_dependent t then f ts else Syntax.const Q $ A $ s
     | _ => f ts;
   fun contract2 (Q,f) = (Q, contract Q f);
   val pairs =