aboutsummaryrefslogtreecommitdiff
path: root/kernel/indTyping.mli
diff options
context:
space:
mode:
authorGaëtan Gilbert2018-11-19 18:17:06 +0100
committerGaëtan Gilbert2019-01-21 13:22:47 +0100
commit70ce3e98991a96f9d7f181a4a6f5b250457f1245 (patch)
treece3c5c63b3b13d470ce08c339f22e10e34566705 /kernel/indTyping.mli
parent5f9a6c17b4353024e7510977a41cfb1de93a0f5f (diff)
Move inductive typecheck to file independent from positivity check.
This is strictly code movement.
Diffstat (limited to 'kernel/indTyping.mli')
-rw-r--r--kernel/indTyping.mli24
1 files changed, 24 insertions, 0 deletions
diff --git a/kernel/indTyping.mli b/kernel/indTyping.mli
new file mode 100644
index 0000000000..b16ada5ee8
--- /dev/null
+++ b/kernel/indTyping.mli
@@ -0,0 +1,24 @@
+(************************************************************************)
+(* * 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) *)
+(************************************************************************)
+
+open Names
+open Constr
+open Environ
+
+val typecheck_inductive :
+ env ->
+ Entries.mutual_inductive_entry ->
+ env * env * rel_context *
+ (Id.t * Id.t list * types array *
+ (rel_context *
+ (bool * types * Univ.Universe.t,
+ Univ.Level.t option list * Univ.Universe.t)
+ Declarations.declaration_arity))
+ array