aboutsummaryrefslogtreecommitdiff
path: root/kernel/term.mli
diff options
context:
space:
mode:
authorherbelin2000-09-12 11:02:30 +0000
committerherbelin2000-09-12 11:02:30 +0000
commit6fcd224c128ae5e81f4cce9d5de1ac45883cfebf (patch)
tree9d5c886b18ca44f3a24de7b58c7dd7ca8bc88eec /kernel/term.mli
parent9248485d71d1c9c1796a22e526e07784493e2008 (diff)
Modification mkAppL; abstraction via kind_of_term; changement dans Reduction
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@597 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/term.mli')
-rw-r--r--kernel/term.mli15
1 files changed, 10 insertions, 5 deletions
diff --git a/kernel/term.mli b/kernel/term.mli
index fe3996c5c6..fa0d076730 100644
--- a/kernel/term.mli
+++ b/kernel/term.mli
@@ -134,7 +134,7 @@ type kindOfTerm =
| IsProd of name * constr * constr
| IsLambda of name * constr * constr
| IsLetIn of name * constr * constr * constr
- | IsAppL of constr * constr list
+ | IsAppL of constr * constr array
| IsEvar of existential
| IsConst of constant
| IsMutInd of inductive
@@ -216,10 +216,11 @@ val mkNamedLambda : identifier -> constr -> constr -> constr
(* [mkLambda_string s t c] constructs $[s:t]c$ *)
val mkLambda_string : string -> constr -> constr -> constr
-(* If $a = [| t_1; \dots; t_n |]$, constructs the application
- $(t_1~\dots~t_n)$. *)
-val mkAppL : constr array -> constr
-val mkAppList : constr -> constr list -> constr
+(* [mkAppL (f,[| t_1; ...; t_n |]] constructs the application
+ $(f~t_1~\dots~t_n)$. *)
+val mkAppL : constr * constr array -> constr
+val mkAppList : constr list -> constr
+val mkAppA : constr array -> constr
(* Constructs a constant *)
(* The array of terms correspond to the variables introduced in the section *)
@@ -307,6 +308,7 @@ val is_Set : constr -> bool
val isprop : constr -> bool
val is_Type : constr -> bool
val iskind : constr -> bool
+val isSort : constr -> bool
val is_existential_oper : sorts oper -> bool
@@ -324,6 +326,9 @@ val strip_outer_cast : constr -> constr
(* Special function, which keep the key casts under Fix and MutCase. *)
val strip_all_casts : constr -> constr
+(* Apply a function letting Casted types in place *)
+val under_casts : (constr -> constr) -> constr -> constr
+
(* Tests if a de Bruijn index *)
val isRel : constr -> bool