src/HOL/String.thy
changeset 81118 9e2eb05cc2b7
parent 81113 6fefd6c602fa
child 81124 6ce0c8d59f5a
--- a/src/HOL/String.thy	Sat Oct 05 15:18:49 2024 +0200
+++ b/src/HOL/String.thy	Sat Oct 05 22:24:24 2024 +0200
@@ -224,7 +224,7 @@
 type_synonym string = "char list"
 
 syntax
-  "_String" :: "str_position \<Rightarrow> string"    (\<open>_\<close>)
+  "_String" :: "str_position \<Rightarrow> string"    (\<open>(\<open>notation=\<open>literal string\<close>\<close>_)\<close>)
 
 ML_file \<open>Tools/string_syntax.ML\<close>