aboutsummaryrefslogtreecommitdiff
path: root/kernel/uGraph.ml
diff options
context:
space:
mode:
authorGaëtan Gilbert2020-01-27 13:29:18 +0100
committerGaëtan Gilbert2020-01-27 13:29:18 +0100
commit458cf1324163821b60ab0b731a60bb1977576d9f (patch)
tree447f35851e86707b4eacc6dc8feebf1e8cf725be /kernel/uGraph.ml
parent506b35913103c17e4d27663aa0f977452d5815b0 (diff)
Small API additions to kernel/univ
- allow viewing the internal representation of uglobal and universe (with universe, this replaces the "map" function. I kept exists and for_all as they felt somewhat convenient) - add universe set and map modules (currently unused but they're natural)
Diffstat (limited to 'kernel/uGraph.ml')
-rw-r--r--kernel/uGraph.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/kernel/uGraph.ml b/kernel/uGraph.ml
index 33336079bb..4d15ce741c 100644
--- a/kernel/uGraph.ml
+++ b/kernel/uGraph.ml
@@ -128,7 +128,7 @@ let enforce_leq_alg u v g =
| exception (UniverseInconsistency _ as e) -> Inr e)
in
(* max(us) <= max(vs) <-> forall u in us, exists v in vs, u <= v *)
- let c = Universe.map (fun u -> Universe.map (fun v -> (u,v)) v) u in
+ let c = List.map (fun u -> List.map (fun v -> (u,v)) (Universe.repr v)) (Universe.repr u) in
let c = List.cartesians enforce_one (Inl (Constraint.empty,g)) c in
(* We pick a best constraint: smallest number of constraints, not an error if possible. *)
let order x y = match x, y with