src/Doc/Isar_Ref/HOL_Specific.thy
changeset 63183 4d04e14d7ab8
parent 63182 b065b4833092
child 63285 e9c777bfd78c
--- a/src/Doc/Isar_Ref/HOL_Specific.thy	Mon May 30 14:15:44 2016 +0200
+++ b/src/Doc/Isar_Ref/HOL_Specific.thy	Mon May 30 20:58:16 2016 +0200
@@ -264,12 +264,11 @@
   \end{matharray}
 
   @{rail \<open>
-    @@{command (HOL) primrec} @{syntax "fixes"} @'where' @{syntax multi_specs}
+    @@{command (HOL) primrec} @{syntax specification}
     ;
-    (@@{command (HOL) fun} | @@{command (HOL) function}) function_opts? \<newline>
-      @{syntax "fixes"} @'where' @{syntax multi_specs}
+    (@@{command (HOL) fun} | @@{command (HOL) function}) opts? @{syntax specification}
     ;
-    function_opts: '(' (('sequential' | 'domintros') + ',') ')'
+    opts: '(' (('sequential' | 'domintros') + ',') ')'
     ;
     @@{command (HOL) termination} @{syntax term}?
     ;
@@ -563,8 +562,8 @@
   \end{matharray}
 
   @{rail \<open>
-    @@{command (HOL) partial_function} '(' @{syntax name} ')' \<newline>
-      @{syntax "fixes"} @'where' @{syntax multi_specs}
+    @@{command (HOL) partial_function} '(' @{syntax name} ')'
+      @{syntax specification}
   \<close>}
 
   \<^descr> @{command (HOL) "partial_function"}~\<open>(mode)\<close> defines