src/HOL/Fun_Def.thy
changeset 67443 3abf6a722518
parent 64591 240a39af9ec4
child 67487 b4e65cd6974a
equal deleted inserted replaced
67442:f075640b8868 67443:3abf6a722518
   293 ML_file "Tools/Function/termination.ML"
   293 ML_file "Tools/Function/termination.ML"
   294 ML_file "Tools/Function/scnp_solve.ML"
   294 ML_file "Tools/Function/scnp_solve.ML"
   295 ML_file "Tools/Function/scnp_reconstruct.ML"
   295 ML_file "Tools/Function/scnp_reconstruct.ML"
   296 ML_file "Tools/Function/fun_cases.ML"
   296 ML_file "Tools/Function/fun_cases.ML"
   297 
   297 
   298 ML_val \<comment> "setup inactive"
   298 ML_val \<comment> \<open>setup inactive\<close>
   299 \<open>
   299 \<open>
   300   Context.theory_map (Function_Common.set_termination_prover
   300   Context.theory_map (Function_Common.set_termination_prover
   301     (K (ScnpReconstruct.decomp_scnp_tac [ScnpSolve.MAX, ScnpSolve.MIN, ScnpSolve.MS])))
   301     (K (ScnpReconstruct.decomp_scnp_tac [ScnpSolve.MAX, ScnpSolve.MIN, ScnpSolve.MS])))
   302 \<close>
   302 \<close>
   303 
   303