src/Pure/Isar/isar_syn.ML
changeset 6108 2c9ed58c30ba
parent 6013 6da9ae6d40f5
child 6196 f9fdb4e29790
equal deleted inserted replaced
6107:1418bc571f23 6108:2c9ed58c30ba
   351 
   351 
   352 
   352 
   353 val proofP = gen_stepP (Scan.option method) false "proof" "backward proof" IsarThy.proof;
   353 val proofP = gen_stepP (Scan.option method) false "proof" "backward proof" IsarThy.proof;
   354 val terminal_proofP = stepP false "by" "terminal backward proof" IsarThy.terminal_proof;
   354 val terminal_proofP = stepP false "by" "terminal backward proof" IsarThy.terminal_proof;
   355 
   355 
   356 val trivial_proofP =
   356 val immediate_proofP =
   357   OuterSyntax.parser false "." "trivial proof"
   357   OuterSyntax.parser false "." "immediate proof"
   358     (Scan.succeed (Toplevel.print o Toplevel.proof IsarThy.trivial_proof));
   358     (Scan.succeed (Toplevel.print o Toplevel.proof IsarThy.immediate_proof));
   359 
   359 
   360 val default_proofP =
   360 val default_proofP =
   361   OuterSyntax.parser false ".." "default proof"
   361   OuterSyntax.parser false ".." "default proof"
   362     (Scan.succeed (Toplevel.print o Toplevel.proof IsarThy.default_proof));
   362     (Scan.succeed (Toplevel.print o Toplevel.proof IsarThy.default_proof));
   363 
   363 
   522   typed_print_translationP, print_ast_translationP,
   522   typed_print_translationP, print_ast_translationP,
   523   token_translationP, oracleP,
   523   token_translationP, oracleP,
   524   (*proof commands*)
   524   (*proof commands*)
   525   theoremP, lemmaP, showP, haveP, assumeP, fixP, letP, thenP, fromP,
   525   theoremP, lemmaP, showP, haveP, assumeP, fixP, letP, thenP, fromP,
   526   factsP, beginP, nextP, qedP, qed_withP, kill_proofP, refineP,
   526   factsP, beginP, nextP, qedP, qed_withP, kill_proofP, refineP,
   527   then_refineP, proofP, terminal_proofP, trivial_proofP,
   527   then_refineP, proofP, terminal_proofP, immediate_proofP,
   528   default_proofP, clear_undoP, undoP, redoP, undosP, redosP, backP,
   528   default_proofP, clear_undoP, undoP, redoP, undosP, redosP, backP,
   529   prevP, upP, topP,
   529   prevP, upP, topP,
   530   (*diagnostic commands*)
   530   (*diagnostic commands*)
   531   print_commandsP, print_theoryP, print_syntaxP, print_attributesP,
   531   print_commandsP, print_theoryP, print_syntaxP, print_attributesP,
   532   print_methodsP, print_theoremsP, print_bindsP, print_lthmsP,
   532   print_methodsP, print_theoremsP, print_bindsP, print_lthmsP,