src/Doc/Isar_Ref/Proof.thy
changeset 60414 f25f2f2ba48c
parent 60406 12cc54fac9b0
child 60448 78f3c67bc35e
equal deleted inserted replaced
60413:0824fd1e9c40 60414:f25f2f2ba48c
   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}) (stmt | statement)
   435      @@{command schematic_corollary}) (stmt | statement)
   436     ;
   436     ;
   437     (@@{command have} | @@{command show} | @@{command hence} | @@{command thus})
   437     (@@{command have} | @@{command show} | @@{command hence} | @@{command thus})
   438       stmt @{syntax for_fixes}
   438       stmt if_prems @{syntax for_fixes}
   439     ;
   439     ;
   440     @@{command print_statement} @{syntax modes}? @{syntax thmrefs}
   440     @@{command print_statement} @{syntax modes}? @{syntax thmrefs}
   441     ;
   441     ;
   442   
   442   
   443     stmt: (@{syntax props} + @'and')
   443     stmt: (@{syntax props} + @'and')
       
   444     ;
       
   445     if_prems: (@'if' stmt)?
   444     ;
   446     ;
   445     statement: @{syntax thmdecl}? (@{syntax_ref "includes"}?) (@{syntax context_elem} *) \<newline>
   447     statement: @{syntax thmdecl}? (@{syntax_ref "includes"}?) (@{syntax context_elem} *) \<newline>
   446       conclusion
   448       conclusion
   447     ;
   449     ;
   448     conclusion: @'shows' stmt | @'obtains' (@{syntax par_name}? obtain_case + '|')
   450     conclusion: @'shows' stmt | @'obtains' (@{syntax par_name}? obtain_case + '|')