src/Doc/Isar_Ref/Misc.thy
changeset 57415 e721124f1b1e
parent 56582 f05b7d6ec592
child 57442 2373b4c61111
equal deleted inserted replaced
57414:fe1be2844fda 57415:e721124f1b1e
    15     @{command_def "find_theorems"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    15     @{command_def "find_theorems"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    16     @{command_def "find_consts"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    16     @{command_def "find_consts"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    17     @{command_def "thm_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    17     @{command_def "thm_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    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_term_bindings"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
    21   \end{matharray}
    21   \end{matharray}
    22 
    22 
    23   @{rail \<open>
    23   @{rail \<open>
    24     (@@{command print_theory} | @@{command print_theorems} | @@{command print_facts}) ('!'?)
    24     (@@{command print_theory} | @@{command print_theorems} | @@{command print_facts}) ('!'?)
    25     ;
    25     ;
    61   
    61   
    62   \item @{command "print_facts"} prints all local facts of the
    62   \item @{command "print_facts"} prints all local facts of the
    63   current context, both named and unnamed ones; the ``@{text "!"}''
    63   current context, both named and unnamed ones; the ``@{text "!"}''
    64   option indicates extra verbosity.
    64   option indicates extra verbosity.
    65   
    65   
    66   \item @{command "print_binds"} prints all term abbreviations
    66   \item @{command "print_term_bindings"} prints all term bindings that
    67   present in the context.
    67   are present in the context.
    68 
    68 
    69   \item @{command "find_theorems"}~@{text criteria} retrieves facts
    69   \item @{command "find_theorems"}~@{text criteria} retrieves facts
    70   from the theory or proof context matching all of given search
    70   from the theory or proof context matching all of given search
    71   criteria.  The criterion @{text "name: p"} selects all theorems
    71   criteria.  The criterion @{text "name: p"} selects all theorems
    72   whose fully qualified name matches pattern @{text p}, which may
    72   whose fully qualified name matches pattern @{text p}, which may