src/Doc/Isar_Ref/Proof_Script.thy
changeset 62969 9f394a16c557
parent 62271 4cfe65cfd369
child 63531 847eefdca90d
equal deleted inserted replaced
62968:4e4738698db4 62969:9f394a16c557
    35     @{command_def "prefer"}\<open>\<^sup>*\<close> & : & \<open>proof \<rightarrow> proof\<close> \\
    35     @{command_def "prefer"}\<open>\<^sup>*\<close> & : & \<open>proof \<rightarrow> proof\<close> \\
    36     @{command_def "back"}\<open>\<^sup>*\<close> & : & \<open>proof \<rightarrow> proof\<close> \\
    36     @{command_def "back"}\<open>\<^sup>*\<close> & : & \<open>proof \<rightarrow> proof\<close> \\
    37   \end{matharray}
    37   \end{matharray}
    38 
    38 
    39   @{rail \<open>
    39   @{rail \<open>
    40     @@{command supply} (@{syntax thmdef}? @{syntax thmrefs} + @'and')
    40     @@{command supply} (@{syntax thmdef}? @{syntax thms} + @'and')
    41     ;
    41     ;
    42     ( @@{command apply} | @@{command apply_end} ) @{syntax method}
    42     ( @@{command apply} | @@{command apply_end} ) @{syntax method}
    43     ;
    43     ;
    44     @@{command defer} @{syntax nat}?
    44     @@{command defer} @{syntax nat}?
    45     ;
    45     ;
   220   \end{matharray}
   220   \end{matharray}
   221 
   221 
   222   @{rail \<open>
   222   @{rail \<open>
   223     (@@{method rule_tac} | @@{method erule_tac} | @@{method drule_tac} |
   223     (@@{method rule_tac} | @@{method erule_tac} | @@{method drule_tac} |
   224       @@{method frule_tac} | @@{method cut_tac}) @{syntax goal_spec}? \<newline>
   224       @@{method frule_tac} | @@{method cut_tac}) @{syntax goal_spec}? \<newline>
   225     (@{syntax named_insts} @{syntax for_fixes} @'in' @{syntax thmref} | @{syntax thmrefs} )
   225     (@{syntax named_insts} @{syntax for_fixes} @'in' @{syntax thm} | @{syntax thms} )
   226     ;
   226     ;
   227     @@{method thin_tac} @{syntax goal_spec}? @{syntax prop} @{syntax for_fixes}
   227     @@{method thin_tac} @{syntax goal_spec}? @{syntax prop} @{syntax for_fixes}
   228     ;
   228     ;
   229     @@{method subgoal_tac} @{syntax goal_spec}? (@{syntax prop} +) @{syntax for_fixes}
   229     @@{method subgoal_tac} @{syntax goal_spec}? (@{syntax prop} +) @{syntax for_fixes}
   230     ;
   230     ;