src/HOL/Decision_Procs/Ferrack.thy
changeset 33063 4d462963a7db
parent 32960 69916a850301
child 33639 603320b93668
equal deleted inserted replaced
33062:542b34b178ec 33063:4d462963a7db
  2071 in fn ct =>
  2071 in fn ct =>
  2072   let 
  2072   let 
  2073     val thy = Thm.theory_of_cterm ct;
  2073     val thy = Thm.theory_of_cterm ct;
  2074     val t = Thm.term_of ct;
  2074     val t = Thm.term_of ct;
  2075     val fs = OldTerm.term_frees t;
  2075     val fs = OldTerm.term_frees t;
  2076     val vs = fs ~~ (0 upto (length fs - 1));
  2076     val vs = map_index swap fs;
  2077     val res = HOLogic.mk_Trueprop (HOLogic.mk_eq (t, term_of_fm vs (@{code linrqe} (fm_of_term vs t))));
  2077     val res = HOLogic.mk_Trueprop (HOLogic.mk_eq (t, term_of_fm vs (@{code linrqe} (fm_of_term vs t))));
  2078   in Thm.cterm_of thy res end
  2078   in Thm.cterm_of thy res end
  2079 end;
  2079 end;
  2080 *}
  2080 *}
  2081 
  2081