aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/constr.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-17 14:26:02 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-17 15:44:38 +0200
commit90d64647d3fd5dbf5c337944dc0038f0b19b8a51 (patch)
treeb33528c72730ec541a75e3d0baaead6789f4dcb9 /kernel/constr.ml
parentd412844753ef25f4431c209f47b97b9fa498297d (diff)
Removing dead code.
Diffstat (limited to 'kernel/constr.ml')
-rw-r--r--kernel/constr.ml6
1 files changed, 1 insertions, 5 deletions
diff --git a/kernel/constr.ml b/kernel/constr.ml
index 9be04c765..b2aa5690b 100644
--- a/kernel/constr.ml
+++ b/kernel/constr.ml
@@ -143,7 +143,6 @@ let mkApp (f, a) =
| App (g, cl) -> App (g, Array.append cl a)
| _ -> App (f, a)
-let out_punivs (a, _) = a
let map_puniverses f (x,u) = (f x, u)
let in_punivs a = (a, Univ.Instance.empty)
@@ -547,9 +546,6 @@ let compare_head_gen_leq eq_universes eq_sorts leq_sorts eq leq t1 t2 =
let rec eq_constr m n =
(m == n) || compare_head_gen (fun _ -> Instance.equal) Sorts.equal eq_constr m n
-(** Strict equality of universe instances. *)
-let compare_constr = compare_head_gen (fun _ -> Instance.equal) Sorts.equal
-
let equal m n = eq_constr m n (* to avoid tracing a recursive fun *)
let eq_constr_univs univs m n =
@@ -989,7 +985,7 @@ module Hsorts =
| Type u -> 2 + Universe.hash u
end)
-let hcons_sorts = Hashcons.simple_hcons Hsorts.generate hcons_univ
+(* let hcons_sorts = Hashcons.simple_hcons Hsorts.generate hcons_univ *)
let hcons_caseinfo = Hashcons.simple_hcons Hcaseinfo.generate hcons_ind
let hcons =