doc-src/IsarRef/Thy/Quick_Reference.thy
changeset 40536 270f47a6d8f8
parent 40535 732f0826f1ba
child 42651 e3fdb7c96be5
equal deleted inserted replaced
40535:732f0826f1ba 40536:270f47a6d8f8
    98 
    98 
    99 text {*
    99 text {*
   100   \begin{tabular}{ll}
   100   \begin{tabular}{ll}
   101     @{command "pr"} & print current state \\
   101     @{command "pr"} & print current state \\
   102     @{command "thm"}~@{text a} & print fact \\
   102     @{command "thm"}~@{text a} & print fact \\
       
   103     @{command "prop"}~@{text \<phi>} & print proposition \\
   103     @{command "term"}~@{text t} & print term \\
   104     @{command "term"}~@{text t} & print term \\
   104     @{command "prop"}~@{text \<phi>} & print meta-level proposition \\
   105     @{command "typ"}~@{text \<tau>} & print type \\
   105     @{command "typ"}~@{text \<tau>} & print meta-level type \\
       
   106   \end{tabular}
   106   \end{tabular}
   107 *}
   107 *}
   108 
   108 
   109 
   109 
   110 section {* Proof methods *}
   110 section {* Proof methods *}