src/Pure/Tools/find_consts.ML
changeset 33301 1fe9fc908ec3
parent 33158 6e3dc0ba2b06
child 35845 e5980f0ad025
equal deleted inserted replaced
33300:939ca97f5a11 33301:1fe9fc908ec3
     9 sig
     9 sig
    10   datatype criterion =
    10   datatype criterion =
    11       Strict of string
    11       Strict of string
    12     | Loose of string
    12     | Loose of string
    13     | Name of string
    13     | Name of string
    14 
       
    15   val find_consts : Proof.context -> (bool * criterion) list -> unit
    14   val find_consts : Proof.context -> (bool * criterion) list -> unit
    16 end;
    15 end;
    17 
    16 
    18 structure FindConsts : FIND_CONSTS =
    17 structure Find_Consts : FIND_CONSTS =
    19 struct
    18 struct
    20 
    19 
    21 (* search criteria *)
    20 (* search criteria *)
    22 
    21 
    23 datatype criterion =
    22 datatype criterion =
   160 
   159 
   161 in
   160 in
   162 
   161 
   163 val _ =
   162 val _ =
   164   OuterSyntax.improper_command "find_consts" "search constants by type pattern" K.diag
   163   OuterSyntax.improper_command "find_consts" "search constants by type pattern" K.diag
   165     (Scan.repeat (((Scan.option P.minus >> is_none) -- criterion))
   164     (Scan.repeat ((Scan.option P.minus >> is_none) -- criterion)
   166       >> (Toplevel.no_timing oo find_consts_cmd));
   165       >> (Toplevel.no_timing oo find_consts_cmd));
   167 
   166 
   168 end;
   167 end;
   169 
   168 
   170 end;
   169 end;