src/HOL/Tools/Sledgehammer/meson_tactic.ML
changeset 37498 b426cbdb5a23
parent 35865 2f8fb5242799
child 37574 b8c1f4c46983
--- a/src/HOL/Tools/Sledgehammer/meson_tactic.ML	Tue Jun 22 13:17:59 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/meson_tactic.ML	Tue Jun 22 14:28:22 2010 +0200
@@ -17,11 +17,11 @@
 open Sledgehammer_Fact_Preprocessor
 
 (*Expand all new definitions of abstraction or Skolem functions in a proof state.*)
-fun is_absko (Const (@{const_name "=="}, _) $ Free (a, _) $ u) =
+fun is_absko (Const (@{const_name "=="}, _) $ Free (a, _) $ _) =
     String.isPrefix skolem_prefix a
   | is_absko _ = false;
 
-fun is_okdef xs (Const (@{const_name "=="}, _) $ t $ u) =   (*Definition of Free, not in certain terms*)
+fun is_okdef xs (Const (@{const_name "=="}, _) $ t $ _) =   (*Definition of Free, not in certain terms*)
       is_Free t andalso not (member (op aconv) xs t)
   | is_okdef _ _ = false