equal
deleted
inserted
replaced
369 ; |
369 ; |
370 @{syntax_def context_elem}: |
370 @{syntax_def context_elem}: |
371 @'fixes' (@{syntax \"fixes\"} + @'and') | |
371 @'fixes' (@{syntax \"fixes\"} + @'and') | |
372 @'constrains' (@{syntax name} '::' @{syntax type} + @'and') | |
372 @'constrains' (@{syntax name} '::' @{syntax type} + @'and') | |
373 @'assumes' (@{syntax props} + @'and') | |
373 @'assumes' (@{syntax props} + @'and') | |
374 @'defines' (@{syntax thmdecl}? @{syntax prop} @{syntax proppat}? + @'and') | |
374 @'defines' (@{syntax thmdecl}? @{syntax prop} @{syntax prop_pat}? + @'and') | |
375 @'notes' (@{syntax thmdef}? @{syntax thmrefs} + @'and') |
375 @'notes' (@{syntax thmdef}? @{syntax thmrefs} + @'and') |
376 "} |
376 "} |
377 |
377 |
378 \begin{description} |
378 \begin{description} |
379 |
379 |