adding remarks after static inspection of the invocation of the SML code generator
--- a/src/HOL/Library/Transitive_Closure_Table.thy Mon Jul 25 23:27:20 2011 +0200
+++ b/src/HOL/Library/Transitive_Closure_Table.thy Tue Jul 26 08:07:00 2011 +0200
@@ -201,7 +201,9 @@
| "test B A"
| "test B C"
-subsubsection {* Invoking with the SML code generator *}
+subsubsection {* Invoking with the (legacy) SML code generator *}
+
+text {* this test can be removed once the SML code generator is deactivated *}
code_module Test
contains
--- a/src/HOL/Proofs/Extraction/Higman.thy Mon Jul 25 23:27:20 2011 +0200
+++ b/src/HOL/Proofs/Extraction/Higman.thy Tue Jul 26 08:07:00 2011 +0200
@@ -408,6 +408,9 @@
end;
*}
+text {* The same story with the legacy SML code generator,
+this can be removed once the code generator is removed. *}
+
code_module Higman
contains
higman = higman_idx
--- a/src/HOL/Proofs/Extraction/Pigeonhole.thy Mon Jul 25 23:27:20 2011 +0200
+++ b/src/HOL/Proofs/Extraction/Pigeonhole.thy Tue Jul 26 08:07:00 2011 +0200
@@ -252,6 +252,10 @@
ML "timeit (@{code test} 500)"
ML "timeit @{code test''}"
+text {* the same story with the legacy SML code generator.
+this can be removed once the code generator is removed.
+*}
+
consts_code
"default :: nat" ("{* 0::nat *}")
"default :: nat \<times> nat" ("{* (0::nat, 0::nat) *}")
--- a/src/HOL/Proofs/Lambda/WeakNorm.thy Mon Jul 25 23:27:20 2011 +0200
+++ b/src/HOL/Proofs/Lambda/WeakNorm.thy Tue Jul 26 08:07:00 2011 +0200
@@ -437,8 +437,10 @@
val ct2' = cterm_of @{theory} (term_of_dB [] (#T (rep_cterm ct2)) dB2);
*}
+
text {*
-The same story again for the SML code generator.
+The same story again for the (legacy) SML code generator.
+This can be removed once the SML code generator is removed.
*}
consts_code