changeset 74101 | d804e93ae9ff |
parent 72611 | c7bc3e70a8c7 |
child 74108 | 3146646a43a7 |
--- a/src/HOL/String.thy Sun Aug 01 23:18:13 2021 +0200 +++ b/src/HOL/String.thy Mon Aug 02 10:01:06 2021 +0000 @@ -3,7 +3,7 @@ section \<open>Character and string types\<close> theory String -imports Enum +imports Enum Bit_Operations Code_Numeral begin subsection \<open>Strings as list of bytes\<close>