From 2e30531e78519a5b9c3773c2524e4fd4759cc5c8 Mon Sep 17 00:00:00 2001 From: Gaƫtan Gilbert Date: Thu, 1 Mar 2018 18:28:36 +0100 Subject: Delayed weak constraints for cumulative inductive types. When comparing 2 irrelevant universes [u] and [v] we add a "weak constraint" [UWeak(u,v)] to the UState. Then at minimization time a weak constraint between unrelated universes where one is flexible causes them to be unified. --- clib/clib.mllib | 1 + clib/orderedType.ml | 35 +++++++++++++++++++++++++++++++++++ clib/orderedType.mli | 19 +++++++++++++++++++ 3 files changed, 55 insertions(+) create mode 100644 clib/orderedType.ml create mode 100644 clib/orderedType.mli (limited to 'clib') diff --git a/clib/clib.mllib b/clib/clib.mllib index 0b5d9826f..c9b4d72fc 100644 --- a/clib/clib.mllib +++ b/clib/clib.mllib @@ -5,6 +5,7 @@ CEphemeron Hashset Hashcons +OrderedType CSet CMap CList diff --git a/clib/orderedType.ml b/clib/orderedType.ml new file mode 100644 index 000000000..922eb76ab --- /dev/null +++ b/clib/orderedType.ml @@ -0,0 +1,35 @@ +(************************************************************************) +(* * The Coq Proof Assistant / The Coq Development Team *) +(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *) +(* t -> int +end + +module Pair (M:S) (N:S) = struct + type t = M.t * N.t + + let compare (a,b) (a',b') = + let i = M.compare a a' in + if Int.equal i 0 then N.compare b b' + else i +end + +module UnorderedPair (M:S) = struct + type t = M.t * M.t + + let reorder (a,b as p) = + if M.compare a b <= 0 then p else (b,a) + + let compare p p' = + let p = reorder p and p' = reorder p' in + let module P = Pair(M)(M) in P.compare p p' +end diff --git a/clib/orderedType.mli b/clib/orderedType.mli new file mode 100644 index 000000000..3578ea0d8 --- /dev/null +++ b/clib/orderedType.mli @@ -0,0 +1,19 @@ +(************************************************************************) +(* * The Coq Proof Assistant / The Coq Development Team *) +(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *) +(* t -> int +end + +module Pair (M:S) (N:S) : S with type t = M.t * N.t + +module UnorderedPair (M:S) : S with type t = M.t * M.t -- cgit v1.2.3