src/HOL/ex/MIR.thy
changeset 29265 5b4247055bd7
parent 29042 d5a5888b8c54
child 29667 53103fc8ffa3
equal deleted inserted replaced
29264:4ea3358fac3f 29265:5b4247055bd7
  5897 
  5897 
  5898 in
  5898 in
  5899   let 
  5899   let 
  5900     val thy = Thm.theory_of_cterm ct;
  5900     val thy = Thm.theory_of_cterm ct;
  5901     val t = Thm.term_of ct;
  5901     val t = Thm.term_of ct;
  5902     val fs = term_frees t;
  5902     val fs = OldTerm.term_frees t;
  5903     val vs = fs ~~ (0 upto (length fs - 1));
  5903     val vs = fs ~~ (0 upto (length fs - 1));
  5904     val qe = if proofs then @{code mirlfrqe} else @{code mircfrqe};
  5904     val qe = if proofs then @{code mirlfrqe} else @{code mircfrqe};
  5905     val t' = (term_of_fm vs o qe o fm_of_term vs) t;
  5905     val t' = (term_of_fm vs o qe o fm_of_term vs) t;
  5906   in (cterm_of thy o HOLogic.mk_Trueprop o HOLogic.mk_eq) (t, t') end
  5906   in (cterm_of thy o HOLogic.mk_Trueprop o HOLogic.mk_eq) (t, t') end
  5907 end;
  5907 end;