src/Doc/Isar_Ref/Inner_Syntax.thy
changeset 80904 05f17df447b6
parent 80773 83d21da2bc59
child 81010 5ea48342e0ae
--- a/src/Doc/Isar_Ref/Inner_Syntax.thy	Thu Sep 19 20:38:34 2024 +0200
+++ b/src/Doc/Isar_Ref/Inner_Syntax.thy	Thu Sep 19 20:56:47 2024 +0200
@@ -391,9 +391,10 @@
     atom: @{syntax short_ident} | @{syntax int} | @{syntax float} | @{syntax cartouche}
   \<close>
 
-  Each @{syntax entry} is a name-value pair: if the value is omitted, it
-  defaults to \<^verbatim>\<open>true\<close> (intended for Boolean properties). The following
-  standard block properties are supported:
+  Each @{syntax entry} is a name-value pair, but the latter is optional. If
+  the value is omitted, the default depends on its type (Boolean: \<^verbatim>\<open>true\<close>,
+  number: \<^verbatim>\<open>1\<close>, otherwise the empty string). The following standard block
+  properties are supported:
 
     \<^item> \<open>indent\<close> (natural number): the block indentation --- the same as for the
     simple syntax without block properties.