src/Doc/IsarRef/Misc.thy
changeset 55112 b1a5d603fd12
parent 55029 61a6bf7d4b02
child 56158 c2c6d560e7b2
equal deleted inserted replaced
55111:5792f5106c40 55112:b1a5d603fd12
    18     @{command_def "unused_thms"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    18     @{command_def "unused_thms"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    19     @{command_def "print_facts"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    19     @{command_def "print_facts"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    20     @{command_def "print_binds"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    20     @{command_def "print_binds"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    21   \end{matharray}
    21   \end{matharray}
    22 
    22 
    23   @{rail "
    23   @{rail \<open>
    24     (@@{command print_theory} | @@{command print_theorems}) ('!'?)
    24     (@@{command print_theory} | @@{command print_theorems}) ('!'?)
    25     ;
    25     ;
    26 
    26 
    27     @@{command find_theorems} ('(' @{syntax nat}? 'with_dups'? ')')? \<newline> (thmcriterion * )
    27     @@{command find_theorems} ('(' @{syntax nat}? 'with_dups'? ')')? \<newline> (thmcriterion * )
    28     ;
    28     ;
    35       ('name' ':' @{syntax nameref} | 'strict' ':' @{syntax type} | @{syntax type})
    35       ('name' ':' @{syntax nameref} | 'strict' ':' @{syntax type} | @{syntax type})
    36     ;
    36     ;
    37     @@{command thm_deps} @{syntax thmrefs}
    37     @@{command thm_deps} @{syntax thmrefs}
    38     ;
    38     ;
    39     @@{command unused_thms} ((@{syntax name} +) '-' (@{syntax name} * ))?
    39     @@{command unused_thms} ((@{syntax name} +) '-' (@{syntax name} * ))?
    40   "}
    40   \<close>}
    41 
    41 
    42   These commands print certain parts of the theory and proof context.
    42   These commands print certain parts of the theory and proof context.
    43   Note that there are some further ones available, such as for the set
    43   Note that there are some further ones available, such as for the set
    44   of rules declared for simplifications.
    44   of rules declared for simplifications.
    45 
    45 
   119     @{command_def "cd"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   119     @{command_def "cd"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   120     @{command_def "pwd"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   120     @{command_def "pwd"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   121     @{command_def "use_thy"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   121     @{command_def "use_thy"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
   122   \end{matharray}
   122   \end{matharray}
   123 
   123 
   124   @{rail "
   124   @{rail \<open>
   125     (@@{command cd} | @@{command use_thy}) @{syntax name}
   125     (@@{command cd} | @@{command use_thy}) @{syntax name}
   126   "}
   126   \<close>}
   127 
   127 
   128   \begin{description}
   128   \begin{description}
   129 
   129 
   130   \item @{command "cd"}~@{text path} changes the current directory
   130   \item @{command "cd"}~@{text path} changes the current directory
   131   of the Isabelle process.
   131   of the Isabelle process.