src/HOL/Proofs/Extraction/Pigeonhole.thy
changeset 46040 4baa475a51e6
parent 44844 a907e541b127
child 52280 0a2371e7ced3
equal deleted inserted replaced
46039:0e8e662013f9 46040:4baa475a51e6
   250 ML "timeit (@{code test} 25)"
   250 ML "timeit (@{code test} 25)"
   251 ML "timeit (@{code test'} 25)"
   251 ML "timeit (@{code test'} 25)"
   252 ML "timeit (@{code test} 500)"
   252 ML "timeit (@{code test} 500)"
   253 ML "timeit @{code test''}"
   253 ML "timeit @{code test''}"
   254 
   254 
   255 text {* the same story with the legacy SML code generator.
       
   256 this can be removed once the code generator is removed.
       
   257 *}
       
   258 
       
   259 consts_code
       
   260   "default :: nat" ("{* 0::nat *}")
       
   261   "default :: nat \<times> nat" ("{* (0::nat, 0::nat) *}")
       
   262 
       
   263 code_module PH
       
   264 contains
       
   265   test = test
       
   266   test' = test'
       
   267   test'' = test''
       
   268 
       
   269 ML "timeit (PH.test 10)"
       
   270 ML "timeit (PH.test' 10)"
       
   271 ML "timeit (PH.test 20)"
       
   272 ML "timeit (PH.test' 20)"
       
   273 ML "timeit (PH.test 25)"
       
   274 ML "timeit (PH.test' 25)"
       
   275 ML "timeit (PH.test 500)"
       
   276 ML "timeit PH.test''"
       
   277 
       
   278 end
   255 end
   279 
   256