aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/btermdn.ml
blob: 1751d41385596f6923513a9209ba4526c2384285 (plain)
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
(************************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team     *)
(* <O___,, *   INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2012     *)
(*   \VV/  **************************************************************)
(*    //   *      This file is distributed under the terms of the       *)
(*         *       GNU Lesser General Public License Version 2.1        *)
(************************************************************************)

open Util
open Term
open Names
open Pattern
open Globnames

(* Discrimination nets with bounded depth.
   See the module dn.ml for further explanations.
   Eduardo (5/8/97). *)

let dnet_depth = ref 8


module Make =
  functor (Z : Map.OrderedType) ->
struct
  open Termdn

  module X = struct
    type t = constr_pattern*int
    let compare = Pervasives.compare (** FIXME *)
  end

 module Y = struct
    type t = term_label
    let compare = compare_term_label
 end

 type 'res lookup_res = 'res Dn.lookup_res = Label of 'res | Nothing | Everything

 module Dn = Dn.Make(X)(Y)(Z)

 type t = Dn.t

  let create = Dn.create

  let decomp =
    let rec decrec acc c = match kind_of_term c with
      | App (f,l) -> decrec (Array.fold_right (fun a l -> a::l) l acc) f
      | Cast (c1,_,_) -> decrec acc c1
      | _ -> (c,acc)
    in
      decrec []

  let constr_val_discr t =
    let c, l = decomp t in
      match kind_of_term c with
      | Ind ind_sp -> Label(GRLabel (IndRef ind_sp),l)
      | Construct cstr_sp -> Label(GRLabel (ConstructRef cstr_sp),l)
      | Var id -> Label(GRLabel (VarRef id),l)
      | Const _ -> Everything
      | _ -> Nothing

  let constr_val_discr_st (idpred,cpred) t =
    let c, l = decomp t in
      match kind_of_term c with
      | Const c -> if Cpred.mem c cpred then Everything else Label(GRLabel (ConstRef c),l)
      | Ind ind_sp -> Label(GRLabel (IndRef ind_sp),l)
      | Construct cstr_sp -> Label(GRLabel (ConstructRef cstr_sp),l)
      | Var id when not (Id.Pred.mem id idpred) -> Label(GRLabel (VarRef id),l)
      | Prod (n, d, c) -> Label(ProdLabel, [d; c])
      | Lambda (n, d, c) -> Label(LambdaLabel, [d; c] @ l)
      | Sort _ -> Label(SortLabel, [])
      | Evar _ -> Everything
      | _ -> Nothing

  let bounded_constr_pat_discr_st st (t,depth) =
    if Int.equal depth 0 then
      None
    else
      match constr_pat_discr_st st t with
	| None -> None
	| Some (c,l) -> Some(c,List.map (fun c -> (c,depth-1)) l)

  let bounded_constr_val_discr_st st (t,depth) =
    if Int.equal depth 0 then
      Nothing
    else
      match constr_val_discr_st st t with
	| Label (c,l) -> Label(c,List.map (fun c -> (c,depth-1)) l)
	| Nothing -> Nothing
	| Everything -> Everything

  let bounded_constr_pat_discr (t,depth) =
    if Int.equal depth 0 then
      None
    else
      match constr_pat_discr t with
	| None -> None
	| Some (c,l) -> Some(c,List.map (fun c -> (c,depth-1)) l)

  let bounded_constr_val_discr (t,depth) =
    if Int.equal depth 0 then
      Nothing
    else
      match constr_val_discr t with
	| Label (c,l) -> Label(c,List.map (fun c -> (c,depth-1)) l)
	| Nothing -> Nothing
	| Everything -> Everything


  let add = function
    | None ->
	(fun dn (c,v) ->
	   Dn.add dn bounded_constr_pat_discr ((c,!dnet_depth),v))
    | Some st ->
	(fun dn (c,v) ->
	   Dn.add dn (bounded_constr_pat_discr_st st) ((c,!dnet_depth),v))

  let rmv = function
    | None ->
	(fun dn (c,v) ->
	   Dn.rmv dn bounded_constr_pat_discr ((c,!dnet_depth),v))
    | Some st ->
	(fun dn (c,v) ->
	 Dn.rmv dn (bounded_constr_pat_discr_st st) ((c,!dnet_depth),v))

  let lookup = function
    | None ->
	(fun dn t ->
	   List.map
	     (fun ((c,_),v) -> (c,v))
	     (Dn.lookup dn bounded_constr_val_discr (t,!dnet_depth)))
    | Some st ->
	(fun dn t ->
	   List.map
	     (fun ((c,_),v) -> (c,v))
	     (Dn.lookup dn (bounded_constr_val_discr_st st) (t,!dnet_depth)))

  let app f dn = Dn.app (fun ((c,_),v) -> f(c,v)) dn

end