doc-src/IsarRef/Thy/Document_Preparation.thy
changeset 46261 b03897da3c90
parent 43618 1c43134ff988
equal deleted inserted replaced
46260:9be4ff2dd91e 46261:b03897da3c90
   153     @{antiquotation_def goals} & : & @{text antiquotation} \\
   153     @{antiquotation_def goals} & : & @{text antiquotation} \\
   154     @{antiquotation_def subgoals} & : & @{text antiquotation} \\
   154     @{antiquotation_def subgoals} & : & @{text antiquotation} \\
   155     @{antiquotation_def prf} & : & @{text antiquotation} \\
   155     @{antiquotation_def prf} & : & @{text antiquotation} \\
   156     @{antiquotation_def full_prf} & : & @{text antiquotation} \\
   156     @{antiquotation_def full_prf} & : & @{text antiquotation} \\
   157     @{antiquotation_def ML} & : & @{text antiquotation} \\
   157     @{antiquotation_def ML} & : & @{text antiquotation} \\
       
   158     @{antiquotation_def ML_op} & : & @{text antiquotation} \\
   158     @{antiquotation_def ML_type} & : & @{text antiquotation} \\
   159     @{antiquotation_def ML_type} & : & @{text antiquotation} \\
   159     @{antiquotation_def ML_struct} & : & @{text antiquotation} \\
   160     @{antiquotation_def ML_struct} & : & @{text antiquotation} \\
   160     @{antiquotation_def "file"} & : & @{text antiquotation} \\
   161     @{antiquotation_def "file"} & : & @{text antiquotation} \\
   161   \end{matharray}
   162   \end{matharray}
   162 
   163 
   195       @@{antiquotation const} options @{syntax term} |
   196       @@{antiquotation const} options @{syntax term} |
   196       @@{antiquotation abbrev} options @{syntax term} |
   197       @@{antiquotation abbrev} options @{syntax term} |
   197       @@{antiquotation typ} options @{syntax type} |
   198       @@{antiquotation typ} options @{syntax type} |
   198       @@{antiquotation type} options @{syntax name} |
   199       @@{antiquotation type} options @{syntax name} |
   199       @@{antiquotation class} options @{syntax name} |
   200       @@{antiquotation class} options @{syntax name} |
   200       @@{antiquotation text} options @{syntax name} |
   201       @@{antiquotation text} options @{syntax name}
       
   202     ;
       
   203     @{syntax antiquotation}:
   201       @@{antiquotation goals} options |
   204       @@{antiquotation goals} options |
   202       @@{antiquotation subgoals} options |
   205       @@{antiquotation subgoals} options |
   203       @@{antiquotation prf} options @{syntax thmrefs} |
   206       @@{antiquotation prf} options @{syntax thmrefs} |
   204       @@{antiquotation full_prf} options @{syntax thmrefs} |
   207       @@{antiquotation full_prf} options @{syntax thmrefs} |
   205       @@{antiquotation ML} options @{syntax name} |
   208       @@{antiquotation ML} options @{syntax name} |
       
   209       @@{antiquotation ML_op} options @{syntax name} |
   206       @@{antiquotation ML_type} options @{syntax name} |
   210       @@{antiquotation ML_type} options @{syntax name} |
   207       @@{antiquotation ML_struct} options @{syntax name} |
   211       @@{antiquotation ML_struct} options @{syntax name} |
   208       @@{antiquotation \"file\"} options @{syntax name}
   212       @@{antiquotation \"file\"} options @{syntax name}
   209     ;
   213     ;
   210     options: '[' (option * ',') ']'
   214     options: '[' (option * ',') ']'
   287   \item @{text "@{full_prf a\<^sub>1 \<dots> a\<^sub>n}"} is like @{text "@{prf a\<^sub>1 \<dots>
   291   \item @{text "@{full_prf a\<^sub>1 \<dots> a\<^sub>n}"} is like @{text "@{prf a\<^sub>1 \<dots>
   288   a\<^sub>n}"}, but prints the full proof terms, i.e.\ also displays
   292   a\<^sub>n}"}, but prints the full proof terms, i.e.\ also displays
   289   information omitted in the compact proof term, which is denoted by
   293   information omitted in the compact proof term, which is denoted by
   290   ``@{text _}'' placeholders there.
   294   ``@{text _}'' placeholders there.
   291   
   295   
   292   \item @{text "@{ML s}"}, @{text "@{ML_type s}"}, and @{text
   296   \item @{text "@{ML s}"}, @{text "@{ML_op s}"}, @{text "@{ML_type
   293   "@{ML_struct s}"} check text @{text s} as ML value, type, and
   297   s}"}, and @{text "@{ML_struct s}"} check text @{text s} as ML value,
   294   structure, respectively.  The source is printed verbatim.
   298   infix operator, type, and structure, respectively.  The source is
       
   299   printed verbatim.
   295 
   300 
   296   \item @{text "@{file path}"} checks that @{text "path"} refers to a
   301   \item @{text "@{file path}"} checks that @{text "path"} refers to a
   297   file (or directory) and prints it verbatim.
   302   file (or directory) and prints it verbatim.
   298 
   303 
   299   \end{description}
   304   \end{description}