src/Doc/Isar_Ref/Outer_Syntax.thy
changeset 61663 63af76397a60
parent 61662 e77def9a63a6
child 62172 7eaeae127955
equal deleted inserted replaced
61662:e77def9a63a6 61663:63af76397a60
   314 subsection \<open>Term patterns and declarations \label{sec:term-decls}\<close>
   314 subsection \<open>Term patterns and declarations \label{sec:term-decls}\<close>
   315 
   315 
   316 text \<open>
   316 text \<open>
   317   Wherever explicit propositions (or term fragments) occur in a proof text,
   317   Wherever explicit propositions (or term fragments) occur in a proof text,
   318   casual binding of schematic term variables may be given specified via
   318   casual binding of schematic term variables may be given specified via
   319   patterns of the form ``\<open>(\<IS> p\<^sub>1 \<dots> p\<^sub>n)\<close>''. This works both for @{syntax
   319   patterns of the form ``\<^theory_text>\<open>(is p\<^sub>1 \<dots> p\<^sub>n)\<close>''. This works both for @{syntax
   320   term} and @{syntax prop}.
   320   term} and @{syntax prop}.
   321 
   321 
   322   @{rail \<open>
   322   @{rail \<open>
   323     @{syntax_def term_pat}: '(' (@'is' @{syntax term} +) ')'
   323     @{syntax_def term_pat}: '(' (@'is' @{syntax term} +) ')'
   324     ;
   324     ;