src/Doc/Codegen/Adaptation.thy
changeset 75647 34cd1d210b92
parent 69690 1fb204399d8d
child 81706 7beb0cf38292
--- a/src/Doc/Codegen/Adaptation.thy	Fri Jul 01 20:47:16 2022 +0200
+++ b/src/Doc/Codegen/Adaptation.thy	Mon Jul 04 07:57:22 2022 +0000
@@ -208,6 +208,10 @@
        containing both \<open>Code_Target_Nat\<close> and
        \<open>Code_Target_Int\<close>.
 
+    \item[\<open>Code_Abstract_Char\<close>] implements type \<^typ>\<open>char\<close> by target language
+       integers, sacrificing pattern patching in exchange for dramatically
+       increased performance for comparisions.
+
     \item[\<^theory>\<open>HOL-Library.IArray\<close>] provides a type \<^typ>\<open>'a iarray\<close>
        isomorphic to lists but implemented by (effectively immutable)
        arrays \emph{in SML only}.