package coq
Formal proof management system
Install
Dune Dependency
Authors
Maintainers
Sources
coq-8.14.0.tar.gz
sha256=b1501d686c21836302191ae30f610cca57fb309214c126518ca009363ad2cd3c
doc/src/ssrsearch_plugin/g_search.ml.html
Source file g_search.ml
1 2 3 4 5 6 7 8 9 10 11 12 13 14 15 16 17 18 19 20 21 22 23 24 25 26 27 28 29 30 31 32 33 34 35 36 37 38 39 40 41 42 43 44 45 46 47 48 49 50 51 52 53 54 55 56 57 58 59 60 61 62 63 64 65 66 67 68 69 70 71 72 73 74 75 76 77 78 79 80 81 82 83 84 85 86 87 88 89 90 91 92 93 94 95 96 97 98 99 100 101 102 103 104 105 106 107 108 109 110 111 112 113 114 115 116 117 118 119 120 121 122 123 124 125 126 127 128 129 130 131 132 133 134 135 136 137 138 139 140 141 142 143 144 145 146 147 148 149 150 151 152 153 154 155 156 157 158 159 160 161 162 163 164 165 166 167 168 169 170 171 172 173 174 175 176 177 178 179 180 181 182 183 184 185 186 187 188 189 190 191 192 193 194 195 196 197 198 199 200 201 202 203 204 205 206 207 208 209 210 211 212 213 214 215 216 217 218 219 220 221 222 223 224 225 226 227 228 229 230 231 232 233 234 235 236 237 238 239 240 241 242 243 244 245 246 247 248 249 250 251 252 253 254 255 256 257 258 259 260 261 262 263 264 265 266 267 268 269 270 271 272 273 274 275 276 277 278 279 280 281 282 283 284 285 286 287 288 289 290 291 292 293 294 295 296 297 298 299 300 301 302 303 304 305 306 307 308 309 310 311 312 313 314 315 316 317 318 319 320 321 322 323 324 325 326 327 328 329 330 331 332 333 334 335 336 337 338 339 340 341 342 343 344 345 346 347 348 349 350 351 352 353 354 355 356 357 358 359 360 361 362 363 364 365 366 367 368 369 370 371 372 373 374 375 376 377 378 379 380 381 382 383 384 385 386 387 388 389 390 391 392 393 394 395 396 397 398 399 400 401 402 403 404 405 406 407 408 409 410 411 412 413 414 415 416 417 418 419 420 421 422 423 424 425 426 427 428 429 430 431 432 433 434 435 436 437 438 439 440 441 442 443 444 445 446 447 448 449 450 451 452 453 454 455 456 457 458 459 460 461 462 463 464 465 466 467 468 469 470 471 472 473 474 475 476 477 478 479 480 481 482 483 484 485 486 487 488 489 490 491 492 493 494 495 496 497 498 499 500 501 502 503 504 505 506
let __coq_plugin_name = "ssrsearch_plugin" let _ = Mltop.add_known_module __coq_plugin_name # 7 "plugins/ssrsearch/g_search.mlg" module CoqConstr = Constr open CoqConstr open Constrexpr open Evar_kinds open Glob_term open Ltac_plugin open Notation_ops open Notation_term open Pcoq.Prim open Pcoq.Constr open Pp open Ppconstr open Printer open Stdarg open Ssreflect_plugin.Ssrprinters open Ssreflect_plugin.Ssrcommon open Ssreflect_plugin.Ssrparser open Termops open Util type raw_glob_search_about_item = | RGlobSearchSubPattern of constr_expr | RGlobSearchString of Loc.t * string * string option let pr_search_item env sigma = function | RGlobSearchString (_,s,_) -> str s | RGlobSearchSubPattern p -> pr_constr_expr env sigma p let wit_ssr_searchitem = add_genarg "ssr_searchitem" pr_search_item let pr_ssr_search_item env sigma _ _ _ = pr_search_item env sigma (* Workaround the notation API that can only print notations *) let is_ident s = try CLexer.check_ident s; true with _ -> false let is_ident_part s = is_ident ("H" ^ s) let interp_search_notation ?loc tag okey = let err msg = CErrors.user_err ?loc ~hdr:"interp_search_notation" msg in let mk_pntn s for_key = let n = String.length s in let s' = Bytes.make (n + 2) ' ' in let rec loop i i' = if i >= n then s', i' - 2 else if s.[i] = ' ' then loop (i + 1) i' else let j = try String.index_from s (i + 1) ' ' with _ -> n in let m = j - i in if s.[i] = '\'' && i < j - 2 && s.[j - 1] = '\'' then (String.blit s (i + 1) s' i' (m - 2); loop (j + 1) (i' + m - 1)) else if for_key && is_ident (String.sub s i m) then (Bytes.set s' i' '_'; loop (j + 1) (i' + 2)) else (String.blit s i s' i' m; loop (j + 1) (i' + m + 1)) in loop 0 1 in let trim_ntn (pntn, m) = (InConstrEntry,Bytes.sub_string pntn 1 (max 0 m)) in let pr_ntn ntn = str "(" ++ Notation.pr_notation ntn ++ str ")" in let pr_and_list pr = function | [x] -> pr x | x :: lx -> pr_list pr_comma pr lx ++ pr_comma () ++ str "and " ++ pr x | [] -> mt () in let pr_sc sc = str (if sc = "" then "independently" else sc) in let pr_scs = function | [""] -> pr_sc "" | scs -> str "in " ++ pr_and_list pr_sc scs in let generator, pr_tag_sc = let ign _ = mt () in match okey with | Some key -> let sc = Notation.find_delimiters_scope ?loc key in let pr_sc s_in = str s_in ++ spc() ++ str sc ++ pr_comma() in Notation.pr_scope ign sc, pr_sc | None -> Notation.pr_scopes ign, ign in let qtag s_in = pr_tag_sc s_in ++ qstring tag ++ spc()in let ptag, ttag = let ptag, m = mk_pntn tag false in if m <= 0 then err (str "empty notation fragment"); ptag, trim_ntn (ptag, m) in let last = ref "" and last_sc = ref "" in let scs = ref [] and ntns = ref [] in let push_sc sc = match !scs with | "" :: scs' -> scs := "" :: sc :: scs' | scs' -> scs := sc :: scs' in let get s _ _ = match !last with | "Scope " -> last_sc := s; last := "" | "Lonely notation" -> last_sc := ""; last := "" | "\"" -> let pntn, m = mk_pntn s true in if String.string_contains ~where:(Bytes.to_string pntn) ~what:(Bytes.to_string ptag) then begin let ntn = trim_ntn (pntn, m) in match !ntns with | [] -> ntns := [ntn]; scs := [!last_sc] | ntn' :: _ when ntn' = ntn -> push_sc !last_sc | _ when ntn = ttag -> ntns := ntn :: !ntns; scs := [!last_sc] | _ :: ntns' when List.mem ntn ntns' -> () | ntn' :: ntns' -> ntns := ntn' :: ntn :: ntns' end; last := "" | _ -> last := s in pp_with (Format.make_formatter get (fun _ -> ())) generator; let ntn = match !ntns with | [] -> err (hov 0 (qtag "in" ++ str "does not occur in any notation")) | ntn :: ntns' when ntn = ttag -> if ntns' <> [] then begin let pr_ntns' = pr_and_list pr_ntn ntns' in Feedback.msg_warning (hov 4 (qtag "In" ++ str "also occurs in " ++ pr_ntns')) end; ntn | [ntn] -> Feedback.msg_notice (hov 4 (qtag "In" ++ str "is part of notation " ++ pr_ntn ntn)); ntn | ntns' -> let e = str "occurs in" ++ spc() ++ pr_and_list pr_ntn ntns' in err (hov 4 (str "ambiguous: " ++ qtag "in" ++ e)) in let (nvars, body), ((_, pat), osc) = match !scs with | [sc] -> Notation.interp_notation ?loc ntn (None, [sc]) | scs' -> try Notation.interp_notation ?loc ntn (None, []) with _ -> let e = pr_ntn ntn ++ spc() ++ str "is defined " ++ pr_scs scs' in err (hov 4 (str "ambiguous: " ++ pr_tag_sc "in" ++ e)) in let sc = Option.default "" osc in let _ = let m_sc = if osc <> None then str "In " ++ str sc ++ pr_comma() else mt() in let ntn_pat = trim_ntn (mk_pntn pat false) in let rbody = glob_constr_of_notation_constr ?loc body in let m_body = hov 0 (Constrextern.without_symbols prl_glob_constr rbody) in let m = m_sc ++ pr_ntn ntn_pat ++ spc () ++ str "denotes " ++ m_body in Feedback.msg_notice (hov 0 m) in if List.length !scs > 1 then let scs' = List.remove (=) sc !scs in let w = pr_ntn ntn ++ str " is also defined " ++ pr_scs scs' in Feedback.msg_warning (hov 4 w) else if String.string_contains ~where:(snd ntn) ~what:" .. " then err (pr_ntn ntn ++ str " is an n-ary notation"); let nvars = List.filter (fun (_,(_,typ)) -> typ = NtnTypeConstr) nvars in let rec sub () = function | NVar x when List.mem_assoc x nvars -> DAst.make ?loc @@ GPatVar (FirstOrderPatVar x) | c -> glob_constr_of_notation_constr_with_binders ?loc (fun _ x t -> (), None, x, Explicit, t) sub () c in let _, npat = Patternops.pattern_of_glob_constr (sub () body) in Search.GlobSearchSubPattern (Vernacexpr.Anywhere,false,npat) let (wit_ssr_search_item, ssr_search_item) = Tacentries.argument_extend ~name:"ssr_search_item" { Tacentries.arg_parsing = Vernacextend.Arg_rules ( [(Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.nterm constr_pattern))) (fun p loc -> # 154 "plugins/ssrsearch/g_search.mlg" RGlobSearchSubPattern p )); (Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.nterm string))) ((Pcoq.Symbol.token (CLexer.terminal "%")))) ((Pcoq.Symbol.nterm preident))) (fun key _ s loc -> # 153 "plugins/ssrsearch/g_search.mlg" RGlobSearchString (loc,s,Some key) )); (Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.nterm string))) (fun s loc -> # 152 "plugins/ssrsearch/g_search.mlg" RGlobSearchString (loc,s,None) ))]); Tacentries.arg_tag = Some (Geninterp.val_tag (Genarg.topwit wit_ssr_searchitem)); Tacentries.arg_intern = Tacentries.ArgInternWit (wit_ssr_searchitem); Tacentries.arg_subst = Tacentries.ArgSubstWit (wit_ssr_searchitem); Tacentries.arg_interp = Tacentries.ArgInterpWit (wit_ssr_searchitem); Tacentries.arg_printer = ((fun env sigma -> # 151 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_item env sigma ), (fun env sigma -> # 151 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_item env sigma ), (fun env sigma -> # 151 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_item env sigma )); } let _ = (wit_ssr_search_item, ssr_search_item) # 157 "plugins/ssrsearch/g_search.mlg" let pr_ssr_search_arg env sigma _ _ _ = let pr_item (b, p) = str (if b then "-" else "") ++ pr_search_item env sigma p in pr_list spc pr_item let (wit_ssr_search_arg, ssr_search_arg) = Tacentries.argument_extend ~name:"ssr_search_arg" { Tacentries.arg_parsing = Vernacextend.Arg_rules ( [( Pcoq.Production.make (Pcoq.Rule.stop) (fun loc -> # 169 "plugins/ssrsearch/g_search.mlg" [] )); ( Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.nterm ssr_search_item))) (Pcoq.Symbol.self)) (fun a p loc -> # 168 "plugins/ssrsearch/g_search.mlg" (true, p) :: a )); ( Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.token (CLexer.terminal "-")))) ((Pcoq.Symbol.nterm ssr_search_item))) (Pcoq.Symbol.self)) (fun a p _ loc -> # 167 "plugins/ssrsearch/g_search.mlg" (false, p) :: a ))]); Tacentries.arg_tag = Some (Geninterp.Val.List (Geninterp.Val.Pair ( (Geninterp.val_tag (Genarg.topwit wit_bool)), (Geninterp.val_tag (Genarg.topwit wit_ssr_searchitem))))); Tacentries.arg_intern = Tacentries.ArgInternWit (Genarg.ListArg (Genarg.PairArg ( (wit_bool), (wit_ssr_searchitem)))); Tacentries.arg_subst = Tacentries.ArgSubstWit (Genarg.ListArg (Genarg.PairArg ( (wit_bool), (wit_ssr_searchitem)))); Tacentries.arg_interp = Tacentries.ArgInterpWit (Genarg.ListArg (Genarg.PairArg ( (wit_bool), (wit_ssr_searchitem)))); Tacentries.arg_printer = ((fun env sigma -> # 166 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_arg env sigma ), (fun env sigma -> # 166 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_arg env sigma ), (fun env sigma -> # 166 "plugins/ssrsearch/g_search.mlg" pr_ssr_search_arg env sigma )); } let _ = (wit_ssr_search_arg, ssr_search_arg) # 172 "plugins/ssrsearch/g_search.mlg" (* Main type conclusion pattern filter *) let rec splay_search_pattern na = function | Pattern.PApp (fp, args) -> splay_search_pattern (na + Array.length args) fp | Pattern.PLetIn (_, _, _, bp) -> splay_search_pattern na bp | Pattern.PRef hr -> hr, na | _ -> CErrors.user_err (Pp.str "no head constant in head search pattern") let push_rels_assum l e = let l = List.map (fun (n,t) -> n, EConstr.Unsafe.to_constr t) l in push_rels_assum l e let coerce_search_pattern_to_sort hpat = let env = Global.env () in let sigma = Evd.(from_env env) in let mkPApp fp n_imps args = let args' = Array.append (Array.make n_imps (Pattern.PMeta None)) args in Pattern.PApp (fp, args') in let hr, na = splay_search_pattern 0 hpat in let dc, ht = let hr, _ = Typeops.type_of_global_in_context env hr (* FIXME *) in Reductionops.splay_prod env sigma (EConstr.of_constr hr) in let np = List.length dc in if np < na then CErrors.user_err (Pp.str "too many arguments in head search pattern") else let hpat' = if np = na then hpat else mkPApp hpat (np - na) [||] in let warn () = Feedback.msg_warning (str "Listing only lemmas with conclusion matching " ++ pr_constr_pattern_env env sigma hpat') in if EConstr.isSort sigma ht then begin warn (); true, hpat' end else let filter_head, coe_path = try let _, cp = Coercionops.lookup_path_to_sort_from (push_rels_assum dc env) sigma ht in warn (); true, cp with _ -> false, [] in let coerce hp coe_index = let coe_ref = coe_index.Coercionops.coe_value in try let n_imps = Option.get (Coercionops.hide_coercion coe_ref) in mkPApp (Pattern.PRef coe_ref) n_imps [|hp|] with Not_found | Option.IsNone -> errorstrm (str "need explicit coercion " ++ pr_global coe_ref ++ spc () ++ str "to interpret head search pattern as type") in filter_head, List.fold_left coerce hpat' coe_path let interp_head_pat hpat = let filter_head, p = coerce_search_pattern_to_sort hpat in let rec loop c = match CoqConstr.kind c with | Cast (c', _, _) -> loop c' | Prod (_, _, c') -> loop c' | LetIn (_, _, _, c') -> loop c' | _ -> let env = Global.env () in let sigma = Evd.from_env env in Constr_matching.is_matching env sigma p (EConstr.of_constr c) in filter_head, loop let all_true _ = true let rec interp_search_about args accu = match args with | [] -> accu | (flag, arg) :: rem -> fun gr kind env typ -> let ans = Search.search_filter arg gr kind env (Evd.from_env env) typ in (if flag then ans else not ans) && interp_search_about rem accu gr kind env typ let interp_search_arg arg = let arg = List.map (fun (x,arg) -> x, match arg with | RGlobSearchString (loc,s,key) -> if is_ident_part s then Search.GlobSearchString s else interp_search_notation ~loc s key | RGlobSearchSubPattern p -> let env = Global.env () in let _, p = Constrintern.intern_constr_pattern env (Evd.from_env env) p in Search.GlobSearchSubPattern (Vernacexpr.Anywhere,false,p)) arg in let hpat, a1 = match arg with | (_, Search.GlobSearchSubPattern (Vernacexpr.Anywhere,false,Pattern.PMeta _)) :: a' -> all_true, a' | (true, Search.GlobSearchSubPattern (Vernacexpr.Anywhere,false,p)) :: a' -> let filter_head, p = interp_head_pat p in if filter_head then p, a' else all_true, arg | (_, (Search.GlobSearchSubPattern (Vernacexpr.(InHyp|InConcl),_,_) |Search.GlobSearchSubPattern (Vernacexpr.Anywhere,true,_))) :: a' -> CErrors.user_err (str "Unsupported.") | _ -> all_true, arg in let is_string = function (_, Search.GlobSearchString _) -> true | _ -> false in let a2, a3 = List.partition is_string a1 in interp_search_about (a2 @ a3) (fun gr kind env typ -> hpat typ) (* Module path postfilter *) let pr_modloc (b, m) = if b then str "-" ++ pr_qualid m else pr_qualid m let wit_ssrmodloc = add_genarg "ssrmodloc" (fun env sigma -> pr_modloc) let pr_ssr_modlocs _ _ _ ml = if ml = [] then str "" else spc () ++ str "in " ++ pr_list spc pr_modloc ml let (wit_ssr_modlocs, ssr_modlocs) = Tacentries.argument_extend ~name:"ssr_modlocs" { Tacentries.arg_parsing = Vernacextend.Arg_rules ( [(Pcoq.Production.make (Pcoq.Rule.stop) (fun loc -> # 276 "plugins/ssrsearch/g_search.mlg" [] ))]); Tacentries.arg_tag = Some (Geninterp.Val.List (Geninterp.val_tag (Genarg.topwit wit_ssrmodloc))); Tacentries.arg_intern = Tacentries.ArgInternWit (Genarg.ListArg (wit_ssrmodloc)); Tacentries.arg_subst = Tacentries.ArgSubstWit (Genarg.ListArg (wit_ssrmodloc)); Tacentries.arg_interp = Tacentries.ArgInterpWit (Genarg.ListArg (wit_ssrmodloc)); Tacentries.arg_printer = ((fun env sigma -> # 275 "plugins/ssrsearch/g_search.mlg" pr_ssr_modlocs ), (fun env sigma -> # 275 "plugins/ssrsearch/g_search.mlg" pr_ssr_modlocs ), (fun env sigma -> # 275 "plugins/ssrsearch/g_search.mlg" pr_ssr_modlocs )); } let _ = (wit_ssr_modlocs, ssr_modlocs) let _ = let modloc = Pcoq.Entry.make "modloc" in let () = assert (Pcoq.Entry.is_empty modloc) in let () = Pcoq.grammar_extend modloc (Pcoq.Fresh (Gramlib.Gramext.First, [(None, None, [Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.nterm global))) (fun m loc -> # 281 "plugins/ssrsearch/g_search.mlg" false, m ); Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.token (Tok.PKEYWORD ("-"))))) ((Pcoq.Symbol.nterm global))) (fun m _ loc -> # 281 "plugins/ssrsearch/g_search.mlg" true, m )])])) in let () = Pcoq.grammar_extend ssr_modlocs (Pcoq.Reuse (None, [Pcoq.Production.make (Pcoq.Rule.next (Pcoq.Rule.next (Pcoq.Rule.stop) ((Pcoq.Symbol.token (Tok.PKEYWORD ("in"))))) ((Pcoq.Symbol.list1 ((Pcoq.Symbol.nterm modloc))))) (fun ml _ loc -> # 282 "plugins/ssrsearch/g_search.mlg" ml )])) in () # 285 "plugins/ssrsearch/g_search.mlg" let interp_modloc mr = let interp_mod (_, qid) = try Nametab.full_name_module qid with Not_found -> CErrors.user_err ?loc:qid.CAst.loc (str "No Module " ++ pr_qualid qid) in let mr_out, mr_in = List.partition fst mr in let interp_bmod b = function | [] -> fun _ _ _ _ _ -> true | rmods -> Search.module_filter (List.map interp_mod rmods, b) in let is_in = interp_bmod false mr_in and is_out = interp_bmod true mr_out in fun gr kind env typ -> is_in gr kind env (Evd.from_env env) typ && is_out gr kind env (Evd.from_env env) typ (* The unified, extended vernacular "Search" command *) let ssrdisplaysearch gr env t = let pr_res = pr_global gr ++ str ":" ++ spc () ++ pr_lconstr_env env Evd.empty t in Feedback.msg_notice (hov 2 pr_res ++ fnl ()) let deprecated_search = CWarnings.create ~name:"deprecated-ssr-search" ~category:"deprecated" (fun () -> Pp.(str"SSReflect's Search command is deprecated.")) let () = Vernacextend.vernac_extend ~command:"SsrSearchPattern" ~classifier:(fun _ -> Vernacextend.classify_as_query) ?entry:None [(Vernacextend.TyML (false, Vernacextend.TyTerminal ("Search", Vernacextend.TyNonTerminal (Extend.TUentry (Genarg.get_arg_tag wit_ssr_search_arg), Vernacextend.TyNonTerminal (Extend.TUentry (Genarg.get_arg_tag wit_ssr_modlocs), Vernacextend.TyNil))), (let coqpp_body a mr () = Vernacextend.VtDefault (fun () -> # 314 "plugins/ssrsearch/g_search.mlg" deprecated_search (); let hpat = interp_search_arg a in let in_mod = interp_modloc mr in let post_filter gr kind env typ = in_mod gr kind env typ && hpat gr kind env typ in let display gr kind env typ = if post_filter gr kind env typ then ssrdisplaysearch gr env typ in let env = Global.env () in Search.generic_search env display ) in fun a mr ?loc ~atts () -> coqpp_body a mr (Attributes.unsupported_attributes atts)), None))]
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>