src/HOL/Decision_Procs/MIR.thy
changeset 33063 4d462963a7db
parent 32960 69916a850301
child 33639 603320b93668
equal deleted inserted replaced
33062:542b34b178ec 33063:4d462963a7db
  5896 in
  5896 in
  5897   let 
  5897   let 
  5898     val thy = Thm.theory_of_cterm ct;
  5898     val thy = Thm.theory_of_cterm ct;
  5899     val t = Thm.term_of ct;
  5899     val t = Thm.term_of ct;
  5900     val fs = OldTerm.term_frees t;
  5900     val fs = OldTerm.term_frees t;
  5901     val vs = fs ~~ (0 upto (length fs - 1));
  5901     val vs = map_index swap fs;
  5902     val qe = if proofs then @{code mirlfrqe} else @{code mircfrqe};
  5902     val qe = if proofs then @{code mirlfrqe} else @{code mircfrqe};
  5903     val t' = (term_of_fm vs o qe o fm_of_term vs) t;
  5903     val t' = (term_of_fm vs o qe o fm_of_term vs) t;
  5904   in (cterm_of thy o HOLogic.mk_Trueprop o HOLogic.mk_eq) (t, t') end
  5904   in (cterm_of thy o HOLogic.mk_Trueprop o HOLogic.mk_eq) (t, t') end
  5905 end;
  5905 end;
  5906 *}
  5906 *}