author | blanchet |
Thu, 28 Jul 2011 11:43:45 +0200 | |
changeset 43998 | a2aa341bc658 |
parent 43997 | 578460971517 |
child 43999 | 04fd92795458 |
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML Thu Jul 28 11:43:45 2011 +0200 +++ b/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML Thu Jul 28 11:43:45 2011 +0200 @@ -537,7 +537,7 @@ Lambda_Lifting.is_quantifier #> fst -fun intentionalize_def (Const (@{const_name All}, _) $ Abs (s, T, t)) = +fun intentionalize_def (Const (@{const_name All}, _) $ Abs (_, _, t)) = intentionalize_def t | intentionalize_def (Const (@{const_name HOL.eq}, _) $ t $ u) = let