diff -r 27f3c10b0b50 -r 4cf66f21b764 src/HOL/String.thy --- a/src/HOL/String.thy Mon Dec 07 10:23:50 2015 +0100 +++ b/src/HOL/String.thy Mon Dec 07 10:38:04 2015 +0100 @@ -115,7 +115,7 @@ by (simp add: nibble_of_nat_def) datatype char = Char nibble nibble - -- "Note: canonical order of character encoding coincides with standard term ordering" + \ "Note: canonical order of character encoding coincides with standard term ordering" syntax "_Char" :: "str_position => char" ("CHR _") @@ -281,7 +281,7 @@ with Char show ?thesis by (simp add: nat_of_char_def add.commute) qed -code_datatype Char -- \drop case certificate for char\ +code_datatype Char \ \drop case certificate for char\ lemma case_char_code [code]: "case_char f c = (let n = nat_of_char c in f (nibble_of_nat (n div 16)) (nibble_of_nat n))"