src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML
changeset 44241 7943b69f0188
parent 43326 47cf4bc789aa
child 45450 dc2236b19a3d
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Wed Aug 17 16:46:58 2011 +0200
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Wed Aug 17 18:05:31 2011 +0200
@@ -914,7 +914,7 @@
             val Ts = binder_types (fastype_of f')
             val bs = map Bound ((length Ts - 1) downto 0)
           in
-            fold (curry absdummy) (rev Ts) (f $ (list_comb (f', bs)))
+            fold_rev absdummy Ts (f $ (list_comb (f', bs)))
           end
         val fs' = map apply_f fs
         val case_c' = Const (case_name, (map fastype_of fs') @ [T] ---> U)
@@ -949,7 +949,7 @@
       val T' = TFree (tname', HOLogic.typeS)
       val U = TFree (uname, HOLogic.typeS)
       val y = Free (yname, U)
-      val f' = absdummy (U --> T', Bound 0 $ y)
+      val f' = absdummy (U --> T') (Bound 0 $ y)
       val th' = Thm.certify_instantiate
         ([(dest_TVar uninst_T, U --> T'), (dest_TVar uninst_T', T')],
          [((fst (dest_Var f), (U --> T') --> T'), f')]) th