src/Doc/Implementation/Logic.thy
changeset 62969 9f394a16c557
parent 62922 96691631c1eb
child 63680 6e1e8b5abbfa
equal deleted inserted replaced
62968:4e4738698db4 62969:9f394a16c557
   169   @{ML_antiquotation_def "nonterminal"} & : & \<open>ML_antiquotation\<close> \\
   169   @{ML_antiquotation_def "nonterminal"} & : & \<open>ML_antiquotation\<close> \\
   170   @{ML_antiquotation_def "typ"} & : & \<open>ML_antiquotation\<close> \\
   170   @{ML_antiquotation_def "typ"} & : & \<open>ML_antiquotation\<close> \\
   171   \end{matharray}
   171   \end{matharray}
   172 
   172 
   173   @{rail \<open>
   173   @{rail \<open>
   174   @@{ML_antiquotation class} nameref
   174   @@{ML_antiquotation class} name
   175   ;
   175   ;
   176   @@{ML_antiquotation sort} sort
   176   @@{ML_antiquotation sort} sort
   177   ;
   177   ;
   178   (@@{ML_antiquotation type_name} |
   178   (@@{ML_antiquotation type_name} |
   179    @@{ML_antiquotation type_abbrev} |
   179    @@{ML_antiquotation type_abbrev} |
   180    @@{ML_antiquotation nonterminal}) nameref
   180    @@{ML_antiquotation nonterminal}) name
   181   ;
   181   ;
   182   @@{ML_antiquotation typ} type
   182   @@{ML_antiquotation typ} type
   183   \<close>}
   183   \<close>}
   184 
   184 
   185   \<^descr> \<open>@{class c}\<close> inlines the internalized class \<open>c\<close> --- as @{ML_type string}
   185   \<^descr> \<open>@{class c}\<close> inlines the internalized class \<open>c\<close> --- as @{ML_type string}
   390   @{ML_antiquotation_def "prop"} & : & \<open>ML_antiquotation\<close> \\
   390   @{ML_antiquotation_def "prop"} & : & \<open>ML_antiquotation\<close> \\
   391   \end{matharray}
   391   \end{matharray}
   392 
   392 
   393   @{rail \<open>
   393   @{rail \<open>
   394   (@@{ML_antiquotation const_name} |
   394   (@@{ML_antiquotation const_name} |
   395    @@{ML_antiquotation const_abbrev}) nameref
   395    @@{ML_antiquotation const_abbrev}) name
   396   ;
   396   ;
   397   @@{ML_antiquotation const} ('(' (type + ',') ')')?
   397   @@{ML_antiquotation const} ('(' (type + ',') ')')?
   398   ;
   398   ;
   399   @@{ML_antiquotation term} term
   399   @@{ML_antiquotation term} term
   400   ;
   400   ;
   699   ;
   699   ;
   700   @@{ML_antiquotation cterm} term
   700   @@{ML_antiquotation cterm} term
   701   ;
   701   ;
   702   @@{ML_antiquotation cprop} prop
   702   @@{ML_antiquotation cprop} prop
   703   ;
   703   ;
   704   @@{ML_antiquotation thm} thmref
   704   @@{ML_antiquotation thm} thm
   705   ;
   705   ;
   706   @@{ML_antiquotation thms} thmrefs
   706   @@{ML_antiquotation thms} thms
   707   ;
   707   ;
   708   @@{ML_antiquotation lemma} ('(' @'open' ')')? ((prop +) + @'and') \<newline>
   708   @@{ML_antiquotation lemma} ('(' @'open' ')')? ((prop +) + @'and') \<newline>
   709     @'by' method method?
   709     @'by' method method?
   710   \<close>}
   710   \<close>}
   711 
   711