src/HOL/Lambda/WeakNorm.thy
changeset 24219 e558fe311376
parent 23810 f5e6932d0500
child 24249 1f60b45c5f97
equal deleted inserted replaced
24218:fbf1646b267c 24219:e558fe311376
   572 text {*
   572 text {*
   573 The same story again for code next generation.
   573 The same story again for code next generation.
   574 *}
   574 *}
   575 
   575 
   576 setup {*
   576 setup {*
   577   CodegenSerializer.add_undefined "SML" "arbitrary" "(raise Fail \"arbitrary\")"
   577   CodeTarget.add_undefined "SML" "arbitrary" "(raise Fail \"arbitrary\")"
   578 *}
   578 *}
   579 
   579 
   580 definition
   580 definition
   581   int :: "nat \<Rightarrow> int" where
   581   int :: "nat \<Rightarrow> int" where
   582   "int \<equiv> of_nat"
   582   "int \<equiv> of_nat"