src/Doc/Isar_Ref/Proof.thy
changeset 59786 0c73c5eb45f7
parent 59785 4e6ab5831cc0
child 59853 4039d8aecda4
equal deleted inserted replaced
59785:4e6ab5831cc0 59786:0c73c5eb45f7
   430   and assumptions, cf.\ \secref{sec:obtain}).
   430   and assumptions, cf.\ \secref{sec:obtain}).
   431 
   431 
   432   @{rail \<open>
   432   @{rail \<open>
   433     (@@{command lemma} | @@{command theorem} | @@{command corollary} |
   433     (@@{command lemma} | @@{command theorem} | @@{command corollary} |
   434      @@{command schematic_lemma} | @@{command schematic_theorem} |
   434      @@{command schematic_lemma} | @@{command schematic_theorem} |
   435      @@{command schematic_corollary}) (goal | longgoal)
   435      @@{command schematic_corollary}) (goal | statement)
   436     ;
   436     ;
   437     (@@{command have} | @@{command show} | @@{command hence} | @@{command thus}) goal
   437     (@@{command have} | @@{command show} | @@{command hence} | @@{command thus}) goal
   438     ;
   438     ;
   439     @@{command print_statement} @{syntax modes}? @{syntax thmrefs}
   439     @@{command print_statement} @{syntax modes}? @{syntax thmrefs}
   440     ;
   440     ;
   441   
   441   
   442     goal: (@{syntax props} + @'and')
   442     goal: (@{syntax props} + @'and')
   443     ;
   443     ;
   444     longgoal: @{syntax thmdecl}? (@{syntax_ref "includes"}?) (@{syntax context_elem} * ) conclusion
   444     statement: @{syntax thmdecl}? (@{syntax_ref "includes"}?) (@{syntax context_elem} *) \<newline>
       
   445       conclusion
   445     ;
   446     ;
   446     conclusion: @'shows' goal | @'obtains' (@{syntax parname}? case + '|')
   447     conclusion: @'shows' goal | @'obtains' (@{syntax parname}? case + '|')
   447     ;
   448     ;
   448     case: (@{syntax vars} + @'and') @'where' (@{syntax props} + @'and')
   449     case: (@{syntax vars} + @'and') @'where' (@{syntax props} + @'and')
   449   \<close>}
   450   \<close>}