src/HOL/ex/Records.thy
changeset 47842 bfc08ce7b7b9
parent 46231 76e32c39dd43
child 51717 9e7d1c139569
--- a/src/HOL/ex/Records.thy	Mon Apr 30 12:14:53 2012 +0200
+++ b/src/HOL/ex/Records.thy	Mon Apr 30 22:18:39 2012 +1000
@@ -324,4 +324,16 @@
 
 export_code foo1 foo3 foo5 foo10 checking SML
 
+text {*
+  Code generation can also be switched off, for instance for very large records
+*}
+
+declare [[record_codegen = false]]
+
+record not_so_large_record =
+  bar520 :: nat
+  bar521 :: "nat * nat"
+
+declare [[record_codegen = true]]
+
 end