aboutsummaryrefslogtreecommitdiff
path: root/kernel/term.ml
diff options
context:
space:
mode:
authorppedrot2012-09-26 19:03:17 +0000
committerppedrot2012-09-26 19:03:17 +0000
commit33509e348a6c9f505a6ebf714d8b142fc9df62a0 (patch)
tree7ad91498f464c99720518571573f4b1661d72c50 /kernel/term.ml
parentae8114a13c48e866c89c165560d34fa862e4ff99 (diff)
Cleaning, renaming obscure functions and documenting in Hashcons.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15834 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/term.ml')
-rw-r--r--kernel/term.ml12
1 files changed, 6 insertions, 6 deletions
diff --git a/kernel/term.ml b/kernel/term.ml
index e54e56f12f..8ab04af24e 100644
--- a/kernel/term.ml
+++ b/kernel/term.ml
@@ -1236,9 +1236,9 @@ let equals_constr t1 t2 =
(** Note that the following Make has the side effect of creating
once and for all the table we'll use for hash-consing all constr *)
-module H = Hashtbl_alt.Make(struct type t = constr let equals = equals_constr end)
+module H = Hashset.Make(struct type t = constr let equal = equals_constr end)
-open Hashtbl_alt.Combine
+open Hashset.Combine
(* [hcons_term hash_consing_functions constr] computes an hash-consed
representation for [constr] using [hash_consing_functions] on
@@ -1369,7 +1369,7 @@ module Hsorts =
struct
type t = sorts
type u = universe -> universe
- let hash_sub huniv = function
+ let hashcons huniv = function
Prop c -> Prop c
| Type u -> Type (huniv u)
let equal s1 s2 =
@@ -1385,7 +1385,7 @@ module Hcaseinfo =
struct
type t = case_info
type u = inductive -> inductive
- let hash_sub hind ci = { ci with ci_ind = hind ci.ci_ind }
+ let hashcons hind ci = { ci with ci_ind = hind ci.ci_ind }
let equal ci ci' =
ci.ci_ind == ci'.ci_ind &&
ci.ci_npar = ci'.ci_npar &&
@@ -1394,8 +1394,8 @@ module Hcaseinfo =
let hash = Hashtbl.hash
end)
-let hcons_sorts = Hashcons.simple_hcons Hsorts.f hcons_univ
-let hcons_caseinfo = Hashcons.simple_hcons Hcaseinfo.f hcons_ind
+let hcons_sorts = Hashcons.simple_hcons Hsorts.generate hcons_univ
+let hcons_caseinfo = Hashcons.simple_hcons Hcaseinfo.generate hcons_ind
let hcons_constr =
hcons_term