diff options
author | Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net> | 2018-03-01 18:28:36 +0100 |
---|---|---|
committer | Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net> | 2018-03-09 16:30:12 +0100 |
commit | 2e30531e78519a5b9c3773c2524e4fd4759cc5c8 (patch) | |
tree | ad7effee5b9ad3904ab84d81e1583d233ae5033a /clib | |
parent | d640b676282285d52ac19038d693080e64eb5ea7 (diff) |
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.
Diffstat (limited to 'clib')
-rw-r--r-- | clib/clib.mllib | 1 | ||||
-rw-r--r-- | clib/orderedType.ml | 35 | ||||
-rw-r--r-- | clib/orderedType.mli | 19 |
3 files changed, 55 insertions, 0 deletions
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 *) +(* <O___,, * (see CREDITS file for the list of authors) *) +(* \VV/ **************************************************************) +(* // * This file is distributed under the terms of the *) +(* * GNU Lesser General Public License Version 2.1 *) +(* * (see LICENSE file for the text of the license) *) +(************************************************************************) + +module type S = +sig + type t + val compare : t -> 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 *) +(* <O___,, * (see CREDITS file for the list of authors) *) +(* \VV/ **************************************************************) +(* // * This file is distributed under the terms of the *) +(* * GNU Lesser General Public License Version 2.1 *) +(* * (see LICENSE file for the text of the license) *) +(************************************************************************) + +module type S = +sig + type t + val compare : t -> 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 |