diff -r 5792f5106c40 -r b1a5d603fd12 src/Doc/IsarRef/Generic.thy --- a/src/Doc/IsarRef/Generic.thy Wed Jan 22 16:03:11 2014 +0100 +++ b/src/Doc/IsarRef/Generic.thy Wed Jan 22 17:02:05 2014 +0100 @@ -34,9 +34,9 @@ @{command_def "print_options"} & : & @{text "context \"} \\ \end{matharray} - @{rail " + @{rail \ @{syntax name} ('=' ('true' | 'false' | @{syntax int} | @{syntax float} | @{syntax name}))? - "} + \} \begin{description} @@ -70,14 +70,14 @@ @{method_def fail} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ (@@{method fold} | @@{method unfold} | @@{method insert}) @{syntax thmrefs} ; (@@{method erule} | @@{method drule} | @@{method frule}) ('(' @{syntax nat} ')')? @{syntax thmrefs} ; (@@{method intro} | @@{method elim}) @{syntax thmrefs}? - "} + \} \begin{description} @@ -136,7 +136,7 @@ @{attribute_def no_vars}@{text "\<^sup>*"} & : & @{text attribute} \\ \end{matharray} - @{rail " + @{rail \ @@{attribute tagged} @{syntax name} @{syntax name} ; @@{attribute untagged} @{syntax name} @@ -146,7 +146,7 @@ (@@{attribute unfolded} | @@{attribute folded}) @{syntax thmrefs} ; @@{attribute rotated} @{syntax int}? - "} + \} \begin{description} @@ -201,11 +201,11 @@ @{method_def split} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ @@{method subst} ('(' 'asm' ')')? \ ('(' (@{syntax nat}+) ')')? @{syntax thmref} ; @@{method split} @{syntax thmrefs} - "} + \} These methods provide low-level facilities for equational reasoning that are intended for specialized applications only. Normally, @@ -304,7 +304,7 @@ @{method_def raw_tactic}@{text "\<^sup>*"} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ (@@{method rule_tac} | @@{method erule_tac} | @@{method drule_tac} | @@{method frule_tac} | @@{method cut_tac} | @@{method thin_tac}) @{syntax goal_spec}? \ ( dynamic_insts @'in' @{syntax thmref} | @{syntax thmrefs} ) @@ -319,7 +319,7 @@ ; dynamic_insts: ((@{syntax name} '=' @{syntax term}) + @'and') - "} + \} \begin{description} @@ -406,7 +406,7 @@ @{method_def simp_all} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ (@@{method simp} | @@{method simp_all}) opt? (@{syntax simpmod} * ) ; @@ -414,7 +414,7 @@ ; @{syntax_def simpmod}: ('add' | 'del' | 'only' | 'split' (() | 'add' | 'del') | 'cong' (() | 'add' | 'del')) ':' @{syntax thmrefs} - "} + \} \begin{description} @@ -608,10 +608,10 @@ @{command_def "print_simpset"}@{text "\<^sup>*"} & : & @{text "context \"} \\ \end{matharray} - @{rail " + @{rail \ (@@{attribute simp} | @@{attribute split} | @@{attribute cong}) (() | 'add' | 'del') - "} + \} \begin{description} @@ -923,13 +923,13 @@ simproc & : & @{text attribute} \\ \end{matharray} - @{rail " + @{rail \ @@{command simproc_setup} @{syntax name} '(' (@{syntax term} + '|') ')' '=' @{syntax text} \ (@'identifier' (@{syntax nameref}+))? ; @@{attribute simproc} (('add' ':')? | 'del' ':') (@{syntax name}+) - "} + \} \begin{description} @@ -1229,12 +1229,12 @@ @{attribute_def simplified} & : & @{text attribute} \\ \end{matharray} - @{rail " + @{rail \ @@{attribute simplified} opt? @{syntax thmrefs}? ; opt: '(' ('no_asm' | 'no_asm_simp' | 'no_asm_use') ')' - "} + \} \begin{description} @@ -1490,13 +1490,13 @@ @{attribute_def swapped} & : & @{text attribute} \\ \end{matharray} - @{rail " + @{rail \ (@@{attribute intro} | @@{attribute elim} | @@{attribute dest}) ('!' | () | '?') @{syntax nat}? ; @@{attribute rule} 'del' ; @@{attribute iff} (((() | 'add') '?'?) | 'del') - "} + \} \begin{description} @@ -1562,9 +1562,9 @@ @{method_def contradiction} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ @@{method rule} @{syntax thmrefs}? - "} + \} \begin{description} @@ -1603,7 +1603,7 @@ @{method_def deepen} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ @@{method blast} @{syntax nat}? (@{syntax clamod} * ) ; @@{method auto} (@{syntax nat} @{syntax nat})? (@{syntax clasimpmod} * ) @@ -1624,7 +1624,7 @@ ('cong' | 'split') (() | 'add' | 'del') | 'iff' (((() | 'add') '?'?) | 'del') | (('intro' | 'elim' | 'dest') ('!' | () | '?') | 'del')) ':' @{syntax thmrefs} - "} + \} \begin{description} @@ -1735,11 +1735,11 @@ @{method_def clarsimp} & : & @{text method} \\ \end{matharray} - @{rail " + @{rail \ (@@{method safe} | @@{method clarify}) (@{syntax clamod} * ) ; @@{method clarsimp} (@{syntax clasimpmod} * ) - "} + \} \begin{description} @@ -1926,13 +1926,13 @@ Generic tools may refer to the information provided by object-logic declarations internally. - @{rail " + @{rail \ @@{command judgment} @{syntax name} '::' @{syntax type} @{syntax mixfix}? ; @@{attribute atomize} ('(' 'full' ')')? ; @@{attribute rule_format} ('(' 'noasm' ')')? - "} + \} \begin{description}