aboutsummaryrefslogtreecommitdiff
path: root/kernel/inferCumulativity.mli
blob: 99d8f0c98daac7ff1ca54100fc73d32eadce9657 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
(************************************************************************)
(*         *   The Coq Proof Assistant / The Coq Development Team       *)
(*  v      *         Copyright INRIA, CNRS and contributors             *)
(* <O___,, * (see version control and CREDITS file for authors & dates) *)
(*   \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)         *)
(************************************************************************)

val infer_inductive
  : env_params:Environ.env
  (** Environment containing the polymorphic universes and the
     parameters. *)
  -> (Univ.Level.t * Univ.Variance.t option) array
  (** Universes whose cumulativity we want to infer or check. *)
  -> Entries.one_inductive_entry list
  (** The inductive block data we want to infer cumulativity for.
      NB: we ignore the template bool and the names, only the terms
      are used. *)
  -> Univ.Variance.t array