src/Pure/Tools/find_consts.ML
author wenzelm
Fri, 27 Feb 2009 15:46:22 +0100
changeset 30142 8d6145694bb5
parent 29895 src/Pure/Isar/find_consts.ML@0e70a29d3e02
child 30143 98a986b02022
permissions -rw-r--r--
moved find_theorems.ML and find_consts.ML to Pure/Tools, collecting main implementation in one place each;

(*  Title:      find_consts.ML
    Author:     Timothy Bourke and Gerwin Klein, NICTA

  Hoogle-like (http://www-users.cs.york.ac.uk/~ndm/hoogle) searching by type
  over constants, but matching is not fuzzy
*)

signature FIND_CONSTS =
sig
  datatype criterion = Strict of string
                     | Loose of string
                     | Name of string

  val default_criteria : (bool * criterion) list ref

  val find_consts : Proof.context -> (bool * criterion) list -> unit
end;

structure FindConsts : FIND_CONSTS =
struct

datatype criterion = Strict of string
                   | Loose of string
                   | Name of string;

val default_criteria = ref [(false, Name ".sko_")];

fun add_tye (_, (_, t)) n = size_of_typ t + n;

fun matches_subtype thy typat = let
    val p = can (fn ty => Sign.typ_match thy (typat, ty) Vartab.empty);

    fun fs [] = false
      | fs (t::ts) = f t orelse fs ts

    and f (t as Type (_, ars)) = p t orelse fs ars
      | f t = p t;
  in f end;

fun check_const p (nm, (ty, _)) = if p (nm, ty)
                                  then SOME (size_of_typ ty)
                                  else NONE;

fun opt_not f (c as (_, (ty, _))) = if is_some (f c)
                                    then NONE else SOME (size_of_typ ty);

fun filter_const (_, NONE) = NONE
  | filter_const (f, (SOME (c, r))) = Option.map
                                        (pair c o ((curry Int.min) r)) (f c);

fun pretty_criterion (b, c) =
  let
    fun prfx s = if b then s else "-" ^ s;
  in
    (case c of
      Strict pat => Pretty.str (prfx "strict: " ^ quote pat)
    | Loose pat => Pretty.str (prfx (quote pat))
    | Name name => Pretty.str (prfx "name: " ^ quote name))
  end;

fun pretty_const ctxt (nm, ty) = let
    val ty' = Logic.unvarifyT ty;
  in
    Pretty.block [Pretty.quote (Pretty.str nm), Pretty.fbrk,
                  Pretty.str "::", Pretty.brk 1,
                  Pretty.quote (Syntax.pretty_typ ctxt ty')]
  end;

fun find_consts ctxt raw_criteria = let
    val start = start_timing ();

    val thy = ProofContext.theory_of ctxt;
    val low_ranking = 10000;

    fun make_pattern crit = ProofContext.read_term_pattern ctxt ("_::" ^ crit)
                            |> type_of;

    fun make_match (Strict arg) =
          let val qty = make_pattern arg; in
            fn (_, (ty, _)) => let
                val tye = Sign.typ_match thy (qty, ty) Vartab.empty;
                val sub_size = Vartab.fold add_tye tye 0;
              in SOME sub_size end handle MATCH => NONE
          end

      | make_match (Loose arg) =
          check_const (matches_subtype thy (make_pattern arg) o snd)
      
      | make_match (Name arg) = check_const (match_string arg o fst);

    fun make_criterion (b, crit) = (if b then I else opt_not) (make_match crit);
    val criteria = map make_criterion ((!default_criteria) @ raw_criteria);

    val (_, consts) = (#constants o Consts.dest o Sign.consts_of) thy;
    fun eval_entry c = foldl filter_const (SOME (c, low_ranking)) criteria;

    val matches = Symtab.fold (cons o eval_entry) consts []
                  |> map_filter I
                  |> sort (rev_order o int_ord o pairself snd)
                  |> map ((apsnd fst) o fst);

    val end_msg = " in " ^
                  (List.nth (String.tokens Char.isSpace (end_timing start), 3))
                  ^ " secs"
  in
    Pretty.big_list "searched for:" (map pretty_criterion raw_criteria)
      :: Pretty.str ""
      :: (Pretty.str o concat)
           (if null matches
            then ["nothing found", end_msg]
            else ["found ", (string_of_int o length) matches,
                  " constants", end_msg, ":"])
      :: Pretty.str ""
      :: map (pretty_const ctxt) matches
    |> Pretty.chunks
    |> Pretty.writeln
  end handle ERROR s => Output.error_msg s



(** command syntax **)

fun find_consts_cmd spec =
  Toplevel.unknown_theory o Toplevel.keep (fn state =>
    find_consts (Proof.context_of (Toplevel.enter_proof_body state)) spec);

local

structure P = OuterParse and K = OuterKeyword;

val criterion =
  P.reserved "strict" |-- P.!!! (P.$$$ ":" |-- P.xname) >> Strict ||
  P.reserved "name" |-- P.!!! (P.$$$ ":" |-- P.xname) >> Name ||
  P.xname >> Loose;

in

val _ =
  OuterSyntax.improper_command "find_consts" "search constants by type pattern" K.diag
    (Scan.repeat (((Scan.option P.minus >> is_none) -- criterion))
      >> (Toplevel.no_timing oo find_consts_cmd));

end;

end;