src/Doc/JEdit/JEdit.thy
changeset 62969 9f394a16c557
parent 62917 eed66ba99bd9
child 63669 256fc20716f2
equal deleted inserted replaced
62968:4e4738698db4 62969:9f394a16c557
  1066   The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Find Theorems\<close> mode retrieves facts from the theory
  1066   The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Find Theorems\<close> mode retrieves facts from the theory
  1067   or proof context matching all of given criteria in the \<^emph>\<open>Find\<close> text field. A
  1067   or proof context matching all of given criteria in the \<^emph>\<open>Find\<close> text field. A
  1068   single criterium has the following syntax:
  1068   single criterium has the following syntax:
  1069 
  1069 
  1070   @{rail \<open>
  1070   @{rail \<open>
  1071     ('-'?) ('name' ':' @{syntax nameref} | 'intro' | 'elim' | 'dest' |
  1071     ('-'?) ('name' ':' @{syntax name} | 'intro' | 'elim' | 'dest' |
  1072       'solves' | 'simp' ':' @{syntax term} | @{syntax term})
  1072       'solves' | 'simp' ':' @{syntax term} | @{syntax term})
  1073   \<close>}
  1073   \<close>}
  1074 
  1074 
  1075   See also the Isar command @{command_ref find_theorems} in @{cite
  1075   See also the Isar command @{command_ref find_theorems} in @{cite
  1076   "isabelle-isar-ref"}.
  1076   "isabelle-isar-ref"}.
  1084   meets all of the given criteria in the \<^emph>\<open>Find\<close> text field. A single
  1084   meets all of the given criteria in the \<^emph>\<open>Find\<close> text field. A single
  1085   criterium has the following syntax:
  1085   criterium has the following syntax:
  1086 
  1086 
  1087   @{rail \<open>
  1087   @{rail \<open>
  1088     ('-'?)
  1088     ('-'?)
  1089       ('name' ':' @{syntax nameref} | 'strict' ':' @{syntax type} | @{syntax type})
  1089       ('name' ':' @{syntax name} | 'strict' ':' @{syntax type} | @{syntax type})
  1090   \<close>}
  1090   \<close>}
  1091 
  1091 
  1092   See also the Isar command @{command_ref find_consts} in @{cite
  1092   See also the Isar command @{command_ref find_consts} in @{cite
  1093   "isabelle-isar-ref"}.
  1093   "isabelle-isar-ref"}.
  1094 \<close>
  1094 \<close>