aboutsummaryrefslogtreecommitdiff
path: root/kernel/vmemitcodes.ml
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2020-09-22 10:44:51 +0200
committerPierre-Marie Pédrot2020-10-21 12:19:02 +0200
commit2b91a8989687e152f7120aa6c907ffeba8495bab (patch)
tree0fd0362eccc5c894b08c65147f0229fcdc8d2814 /kernel/vmemitcodes.ml
parent8f16b1c5b97411b7ea88279699f0f410f1c77723 (diff)
Deprecate the non-qualified equality functions on kerpairs.
This allows to quickly spot the parts of the code that rely on the canonical ordering. When possible we directly introduce the quotient-aware versions.
Diffstat (limited to 'kernel/vmemitcodes.ml')
-rw-r--r--kernel/vmemitcodes.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/kernel/vmemitcodes.ml b/kernel/vmemitcodes.ml
index ec8601edc9..42908a7363 100644
--- a/kernel/vmemitcodes.ml
+++ b/kernel/vmemitcodes.ml
@@ -36,7 +36,7 @@ let eq_reloc_info r1 r2 = match r1, r2 with
| Reloc_annot _, _ -> false
| Reloc_const c1, Reloc_const c2 -> eq_structured_constant c1 c2
| Reloc_const _, _ -> false
-| Reloc_getglobal c1, Reloc_getglobal c2 -> Constant.equal c1 c2
+| Reloc_getglobal c1, Reloc_getglobal c2 -> Constant.CanOrd.equal c1 c2
| Reloc_getglobal _, _ -> false
| Reloc_proj_name p1, Reloc_proj_name p2 -> Projection.Repr.equal p1 p2
| Reloc_proj_name _, _ -> false
@@ -48,7 +48,7 @@ let hash_reloc_info r =
match r with
| Reloc_annot sw -> combinesmall 1 (hash_annot_switch sw)
| Reloc_const c -> combinesmall 2 (hash_structured_constant c)
- | Reloc_getglobal c -> combinesmall 3 (Constant.hash c)
+ | Reloc_getglobal c -> combinesmall 3 (Constant.CanOrd.hash c)
| Reloc_proj_name p -> combinesmall 4 (Projection.Repr.hash p)
| Reloc_caml_prim p -> combinesmall 5 (CPrimitives.hash p)