src/HOL/Tools/Function/lexicographic_order.ML
changeset 60781 2da59cdf531c
parent 60752 b48830b670a1
child 67149 e61557884799
equal deleted inserted replaced
60780:7e2c8a63a8f8 60781:2da59cdf531c
   199                   Pretty.quote (Syntax.pretty_term ctxt relation)])
   199                   Pretty.quote (Syntax.pretty_term ctxt relation)])
   200             else ()
   200             else ()
   201   
   201   
   202         in (* 4: proof reconstruction *)
   202         in (* 4: proof reconstruction *)
   203           st |>
   203           st |>
   204           (PRIMITIVE (cterm_instantiate [apply2 (Thm.cterm_of ctxt) (rel, relation)])
   204           (PRIMITIVE (infer_instantiate ctxt [(#1 (dest_Var rel), Thm.cterm_of ctxt relation)])
   205             THEN (REPEAT (resolve_tac ctxt @{thms wf_mlex} 1))
   205             THEN (REPEAT (resolve_tac ctxt @{thms wf_mlex} 1))
   206             THEN (resolve_tac ctxt @{thms wf_empty} 1)
   206             THEN (resolve_tac ctxt @{thms wf_empty} 1)
   207             THEN EVERY (map (prove_row_tac ctxt) clean_table))
   207             THEN EVERY (map (prove_row_tac ctxt) clean_table))
   208         end
   208         end
   209   end) 1 st;
   209   end) 1 st;