src/HOL/Nitpick_Examples/Mono_Nits.thy
changeset 33224 f93390060bbe
parent 33197 de6285ebcc05
child 33564 e61ad1690c11
equal deleted inserted replaced
33223:1711610c5b7d 33224:f93390060bbe
    12 begin
    12 begin
    13 
    13 
    14 ML {*
    14 ML {*
    15 exception FAIL
    15 exception FAIL
    16 
    16 
    17 val defs = NitpickHOL.all_axioms_of @{theory} |> #1
    17 val defs = Nitpick_HOL.all_axioms_of @{theory} |> #1
    18 val def_table = NitpickHOL.const_def_table @{context} defs
    18 val def_table = Nitpick_HOL.const_def_table @{context} defs
    19 val ext_ctxt =
    19 val ext_ctxt =
    20   {thy = @{theory}, ctxt = @{context}, max_bisim_depth = ~1, boxes = [],
    20   {thy = @{theory}, ctxt = @{context}, max_bisim_depth = ~1, boxes = [],
    21    user_axioms = NONE, debug = false, wfs = [], destroy_constrs = false,
    21    user_axioms = NONE, debug = false, wfs = [], destroy_constrs = false,
    22    specialize = false, skolemize = false, star_linear_preds = false,
    22    specialize = false, skolemize = false, star_linear_preds = false,
    23    uncurry = false, fast_descrs = false, tac_timeout = NONE, evals = [],
    23    uncurry = false, fast_descrs = false, tac_timeout = NONE, evals = [],