aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/univ.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2018-02-12 14:46:05 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2018-02-15 18:02:14 +0100
commitd6ca9b2f71bced8711b184400fa7e80061497fd7 (patch)
tree7d7591a2a1a9cf6e9bb0202e95c68902dae934b2 /kernel/univ.mli
parent8dd6d091ffbfa237f7266eeca60187263a9b521f (diff)
Adding a sanity check on inductive variance subtyping.
Diffstat (limited to 'kernel/univ.mli')
-rw-r--r--kernel/univ.mli3
1 files changed, 3 insertions, 0 deletions
diff --git a/kernel/univ.mli b/kernel/univ.mli
index c45ebe21c..74d1bfd3a 100644
--- a/kernel/univ.mli
+++ b/kernel/univ.mli
@@ -253,6 +253,9 @@ sig
A'] as opposed to [A' <= A]. *)
type t = Irrelevant | Covariant | Invariant
+ (** [check_subtype x y] holds if variance [y] is also an instance of [x] *)
+ val check_subtype : t -> t -> bool
+
val sup : t -> t -> t
val pr : t -> Pp.t