changeset 74309 | 42523fbf643b |
parent 74108 | 3146646a43a7 |
child 75085 | ccc3a72210e6 |
--- a/src/HOL/String.thy Mon Sep 13 13:30:39 2021 +0200 +++ b/src/HOL/String.thy Mon Sep 13 14:18:24 2021 +0000 @@ -121,7 +121,7 @@ lemma char_of_nat [simp]: \<open>char_of (of_nat n) = char_of n\<close> - by (simp add: char_of_def String.char_of_def drop_bit_of_nat bit_simps) + by (simp add: char_of_def String.char_of_def drop_bit_of_nat bit_simps possible_bit_def) end