src/HOL/Library/Code_Test.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 77811 ae9e6218443d
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
   140 definition yxml_string_of_term :: "Code_Evaluation.term \<Rightarrow> yxml_of_term"
   140 definition yxml_string_of_term :: "Code_Evaluation.term \<Rightarrow> yxml_of_term"
   141 where "yxml_string_of_term = yxml_string_of_body \<circ> xml_of_term"
   141 where "yxml_string_of_term = yxml_string_of_body \<circ> xml_of_term"
   142 
   142 
   143 subsection \<open>Test engine and drivers\<close>
   143 subsection \<open>Test engine and drivers\<close>
   144 
   144 
   145 ML_file "code_test.ML"
   145 ML_file \<open>code_test.ML\<close>
   146 
   146 
   147 end
   147 end