src/HOL/Nitpick_Examples/Mono_Nits.thy
changeset 35385 29f81babefd7
parent 35339 34819133c75e
child 35386 45a4e19d3ebd
--- a/src/HOL/Nitpick_Examples/Mono_Nits.thy	Thu Feb 25 10:08:44 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Mono_Nits.thy	Thu Feb 25 16:33:39 2010 +0100
@@ -30,8 +30,7 @@
    special_funs = Unsynchronized.ref [], unrolled_preds = Unsynchronized.ref [],
    wf_cache = Unsynchronized.ref [], constr_cache = Unsynchronized.ref []}
 (* term -> bool *)
-val is_mono = Nitpick_Mono.formulas_monotonic hol_ctxt false @{typ 'a}
-                                              Nitpick_Mono.Plus [] []
+val is_mono = Nitpick_Mono.formulas_monotonic hol_ctxt false @{typ 'a} [] []
 fun is_const t =
   let val T = fastype_of t in
     is_mono (Logic.mk_implies (Logic.mk_equals (Free ("dummyP", T), t),