doc-src/IsarRef/Thy/Misc.thy
changeset 29893 defab1c6a6b5
parent 28779 698960f08652
child 29894 e0e3aa62d9d3
equal deleted inserted replaced
29892:4a396c7a77b5 29893:defab1c6a6b5
    26     ;
    26     ;
    27 
    27 
    28     'find\_theorems' (('(' (nat)? ('with\_dups')? ')')?) (criterion *)
    28     'find\_theorems' (('(' (nat)? ('with\_dups')? ')')?) (criterion *)
    29     ;
    29     ;
    30     criterion: ('-'?) ('name' ':' nameref | 'intro' | 'elim' | 'dest' |
    30     criterion: ('-'?) ('name' ':' nameref | 'intro' | 'elim' | 'dest' |
    31       'simp' ':' term | term)
    31       'solves' | 'simp' ':' term | term)
    32     ;
    32     ;
    33     'thm\_deps' thmrefs
    33     'thm\_deps' thmrefs
    34     ;
    34     ;
    35   \end{rail}
    35   \end{rail}
    36 
    36 
    61   criteria.  The criterion @{text "name: p"} selects all theorems
    61   criteria.  The criterion @{text "name: p"} selects all theorems
    62   whose fully qualified name matches pattern @{text p}, which may
    62   whose fully qualified name matches pattern @{text p}, which may
    63   contain ``@{text "*"}'' wildcards.  The criteria @{text intro},
    63   contain ``@{text "*"}'' wildcards.  The criteria @{text intro},
    64   @{text elim}, and @{text dest} select theorems that match the
    64   @{text elim}, and @{text dest} select theorems that match the
    65   current goal as introduction, elimination or destruction rules,
    65   current goal as introduction, elimination or destruction rules,
    66   respectively.  The criterion @{text "simp: t"} selects all rewrite
    66   respectively.  The criteria @{text "solves"} returns all rules
    67   rules whose left-hand side matches the given term.  The criterion
    67   that would directly solve the current goal.  The criterion
    68   term @{text t} selects all theorems that contain the pattern @{text
    68   @{text "simp: t"} selects all rewrite rules whose left-hand side
    69   t} -- as usual, patterns may contain occurrences of the dummy
    69   matches the given term.  The criterion term @{text t} selects all
    70   ``@{text _}'', schematic variables, and type constraints.
    70   theorems that contain the pattern @{text t} -- as usual, patterns
       
    71   may contain occurrences of the dummy ``@{text _}'', schematic
       
    72   variables, and type constraints.
    71   
    73   
    72   Criteria can be preceded by ``@{text "-"}'' to select theorems that
    74   Criteria can be preceded by ``@{text "-"}'' to select theorems that
    73   do \emph{not} match. Note that giving the empty list of criteria
    75   do \emph{not} match. Note that giving the empty list of criteria
    74   yields \emph{all} currently known facts.  An optional limit for the
    76   yields \emph{all} currently known facts.  An optional limit for the
    75   number of printed facts may be given; the default is 40.  By
    77   number of printed facts may be given; the default is 40.  By