src/HOL/Tools/Nitpick/nitpick_model.ML
changeset 41871 394eef237bd1
parent 41803 ef13e3b7cbaf
child 41875 e3cd0dce9b1a
--- a/src/HOL/Tools/Nitpick/nitpick_model.ML	Wed Mar 02 13:09:57 2011 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick_model.ML	Wed Mar 02 14:50:16 2011 +0100
@@ -862,8 +862,8 @@
 fun reconstruct_hol_model {show_datatypes, show_consts}
         ({hol_ctxt = {thy, ctxt, max_bisim_depth, boxes, stds, wfs, user_axioms,
                       debug, whacks, binary_ints, destroy_constrs, specialize,
-                      star_linear_preds, preconstrs, tac_timeout, evals,
-                      case_names, def_tables, nondef_table, user_nondefs,
+                      star_linear_preds, total_consts, preconstrs, tac_timeout,
+                      evals, case_names, def_tables, nondef_table, user_nondefs,
                       simp_table, psimp_table, choice_spec_table, intro_table,
                       ground_thm_table, ersatz_table, skolems, special_funs,
                       unrolled_preds, wf_cache, constr_cache}, binarize,
@@ -879,15 +879,16 @@
        stds = stds, wfs = wfs, user_axioms = user_axioms, debug = debug,
        whacks = whacks, binary_ints = binary_ints,
        destroy_constrs = destroy_constrs, specialize = specialize,
-       star_linear_preds = star_linear_preds, preconstrs = preconstrs,
-       tac_timeout = tac_timeout, evals = evals, case_names = case_names,
-       def_tables = def_tables, nondef_table = nondef_table,
-       user_nondefs = user_nondefs, simp_table = simp_table,
-       psimp_table = psimp_table, choice_spec_table = choice_spec_table,
-       intro_table = intro_table, ground_thm_table = ground_thm_table,
-       ersatz_table = ersatz_table, skolems = skolems,
-       special_funs = special_funs, unrolled_preds = unrolled_preds,
-       wf_cache = wf_cache, constr_cache = constr_cache}
+       star_linear_preds = star_linear_preds, total_consts = total_consts,
+       preconstrs = preconstrs, tac_timeout = tac_timeout, evals = evals,
+       case_names = case_names, def_tables = def_tables,
+       nondef_table = nondef_table, user_nondefs = user_nondefs,
+       simp_table = simp_table, psimp_table = psimp_table,
+       choice_spec_table = choice_spec_table, intro_table = intro_table,
+       ground_thm_table = ground_thm_table, ersatz_table = ersatz_table,
+       skolems = skolems, special_funs = special_funs,
+       unrolled_preds = unrolled_preds, wf_cache = wf_cache,
+       constr_cache = constr_cache}
     val scope =
       {hol_ctxt = hol_ctxt, binarize = binarize, card_assigns = card_assigns,
        bits = bits, bisim_depth = bisim_depth, datatypes = datatypes, ofs = ofs}