src/HOL/Tools/Nitpick/nitpick_preproc.ML
changeset 35078 6fd1052fe463
parent 35070 96136eb6218f
child 35079 592edca1dfb3
--- a/src/HOL/Tools/Nitpick/nitpick_preproc.ML	Tue Feb 09 16:05:49 2010 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick_preproc.ML	Tue Feb 09 16:07:51 2010 +0100
@@ -943,7 +943,7 @@
                             |> map Logic.mk_equals,
                         Logic.mk_equals (list_comb (Const x1, bounds1 @ args1),
                                          list_comb (Const x2, bounds2 @ args2)))
-    |> Refute.close_form (* TODO: needed? *)
+    |> close_form (* TODO: needed? *)
   end
 
 (* hol_context -> styp list -> term list *)
@@ -1391,7 +1391,7 @@
     val skolem_depth = if skolemize then 4 else ~1
     val (((def_ts, nondef_ts), (got_all_mono_user_axioms, no_poly_user_axioms)),
          core_t) = t |> unfold_defs_in_term hol_ctxt
-                     |> Refute.close_form
+                     |> close_form
                      |> skolemize_term_and_more hol_ctxt skolem_depth
                      |> specialize_consts_in_term hol_ctxt 0
                      |> `(axioms_for_term hol_ctxt)
@@ -1420,7 +1420,7 @@
       #> simplify_constrs_and_sels thy
       #> distribute_quantifiers
       #> push_quantifiers_inward thy
-      #> not core ? Refute.close_form
+      #> close_form
       #> Term.map_abs_vars shortest_name
   in
     (((map (do_rest true false) def_ts, map (do_rest false false) nondef_ts),