aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2019-06-04 10:35:14 +0200
committerPierre-Marie Pédrot2019-06-04 11:16:17 +0200
commit1cdfb1f9270e399a784b346c3f8d6abbc4477552 (patch)
treef11a76b43b4ea825287d22ae15e8d0fe50968d50 /kernel
parent0f54a91eac98baf076d8be8f52bccdb1de17ea46 (diff)
Remove the discharge segment from vo files.
Since the introduction of delayed section substitution, the opaque table was already containing the same information.
Diffstat (limited to 'kernel')
-rw-r--r--kernel/opaqueproof.ml23
-rw-r--r--kernel/opaqueproof.mli1
2 files changed, 11 insertions, 13 deletions
diff --git a/kernel/opaqueproof.ml b/kernel/opaqueproof.ml
index 02d8ff0672..e18b726111 100644
--- a/kernel/opaqueproof.ml
+++ b/kernel/opaqueproof.ml
@@ -130,21 +130,20 @@ module FMap = Future.UUIDMap
let dump ?(except = Future.UUIDSet.empty) { opaque_val = otab; opaque_len = n; _ } =
let opaque_table = Array.make n ([], 0, None) in
- let disch_table = Array.make n [] in
let f2t_map = ref FMap.empty in
let iter n (univs, d, cu) =
let uid = Future.uuid cu in
let () = f2t_map := FMap.add (Future.uuid cu) n !f2t_map in
- if Future.is_val cu then
- let (c, _) = Future.force cu in
- opaque_table.(n) <- (d, univs, Some c)
- else if Future.UUIDSet.mem uid except then
- (* Only monomorphic constraints can be delayed currently *)
- let () = assert (Int.equal univs 0) in
- disch_table.(n) <- d
- else
- CErrors.anomaly
- Pp.(str"Proof object "++int n++str" is not checked nor to be checked")
+ let c =
+ if Future.is_val cu then
+ let (c, _) = Future.force cu in
+ Some c
+ else if Future.UUIDSet.mem uid except then None
+ else
+ CErrors.anomaly
+ Pp.(str"Proof object "++int n++str" is not checked nor to be checked")
+ in
+ opaque_table.(n) <- (d, univs, c)
in
let () = Int.Map.iter iter otab in
- opaque_table, disch_table, !f2t_map
+ opaque_table, !f2t_map
diff --git a/kernel/opaqueproof.mli b/kernel/opaqueproof.mli
index 41f5ebb6b3..6e275649cd 100644
--- a/kernel/opaqueproof.mli
+++ b/kernel/opaqueproof.mli
@@ -66,5 +66,4 @@ val join_opaque : ?except:Future.UUIDSet.t -> opaquetab -> opaque -> unit
val dump : ?except:Future.UUIDSet.t -> opaquetab ->
(cooking_info list * int * Constr.t option) array *
- cooking_info list array *
int Future.UUIDMap.t