aboutsummaryrefslogtreecommitdiffhomepage
path: root/intf/evar_kinds.mli
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-29 11:08:26 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-29 11:08:26 +0000
commit45038a0bfd5621153ba0dd4b6e06755fd15da1e3 (patch)
tree8a30a206d390e1b7450889189596641e5026ee46 /intf/evar_kinds.mli
parent3854ae16ffbaf56b90fbb85bcce3d92cd65ea6a6 (diff)
Evar_kinds.mli containing former Evd.hole_kind, avoid deps on Evd
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15371 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'intf/evar_kinds.mli')
-rw-r--r--intf/evar_kinds.mli29
1 files changed, 29 insertions, 0 deletions
diff --git a/intf/evar_kinds.mli b/intf/evar_kinds.mli
new file mode 100644
index 000000000..fae83ee95
--- /dev/null
+++ b/intf/evar_kinds.mli
@@ -0,0 +1,29 @@
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2010 *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
+
+open Names
+open Libnames
+
+(** The kinds of existential variable *)
+
+(** Should the obligation be defined (opaque or transparent (default)) or
+ defined transparent and expanded in the term? *)
+
+type obligation_definition_status = Define of bool | Expand
+
+type t =
+ | ImplicitArg of global_reference * (int * identifier option)
+ * bool (** Force inference *)
+ | BinderType of name
+ | QuestionMark of obligation_definition_status
+ | CasesType
+ | InternalHole
+ | TomatchTypeParameter of inductive * int
+ | GoalEvar
+ | ImpossibleCase
+ | MatchingVar of bool * identifier