src/HOL/Code_Setup.thy
changeset 24844 98c006a30218
parent 24835 8c26128f8997
child 25534 d0b74fdd6067
--- a/src/HOL/Code_Setup.thy	Thu Oct 04 19:46:09 2007 +0200
+++ b/src/HOL/Code_Setup.thy	Thu Oct 04 19:54:44 2007 +0200
@@ -127,11 +127,6 @@
 
 lemmas [code func] = Let_def if_True if_False
 
-setup {*
-  CodePackage.add_appconst (@{const_name Let}, CodePackage.appgen_let)
-  #> CodePackage.add_appconst (@{const_name If}, CodePackage.appgen_if)
-*}
-
 
 subsection {* Evaluation oracle *}
 
@@ -160,5 +155,4 @@
       THEN' resolve_tac [TrueI, refl]))
 *} "solve goal by normalization"
 
-
 end