src/HOL/Decision_Procs/ferrack_tac.ML
changeset 59621 291934bac95e
parent 59582 0fbed69ff081
child 59629 0d77c51b5040
equal deleted inserted replaced
59620:92d7d8e4f1bf 59621:291934bac95e
    53     val thy = Proof_Context.theory_of ctxt
    53     val thy = Proof_Context.theory_of ctxt
    54     (* Transform the term*)
    54     (* Transform the term*)
    55     val (t,np,nh) = prepare_for_linr q g
    55     val (t,np,nh) = prepare_for_linr q g
    56     (* Some simpsets for dealing with mod div abs and nat*)
    56     (* Some simpsets for dealing with mod div abs and nat*)
    57     val simpset0 = put_simpset HOL_basic_ss ctxt addsimps comp_arith
    57     val simpset0 = put_simpset HOL_basic_ss ctxt addsimps comp_arith
    58     val ct = Thm.cterm_of thy (HOLogic.mk_Trueprop t)
    58     val ct = Thm.global_cterm_of thy (HOLogic.mk_Trueprop t)
    59     (* Theorem for the nat --> int transformation *)
    59     (* Theorem for the nat --> int transformation *)
    60    val pre_thm = Seq.hd (EVERY
    60    val pre_thm = Seq.hd (EVERY
    61       [simp_tac simpset0 1,
    61       [simp_tac simpset0 1,
    62        TRY (simp_tac (put_simpset ferrack_ss ctxt) 1)]
    62        TRY (simp_tac (put_simpset ferrack_ss ctxt) 1)]
    63       (Thm.trivial ct))
    63       (Thm.trivial ct))