aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
Diffstat (limited to 'kernel')
-rw-r--r--kernel/term.ml3
-rw-r--r--kernel/term.mli1
2 files changed, 1 insertions, 3 deletions
diff --git a/kernel/term.ml b/kernel/term.ml
index 99e41ae56c..a4adad7626 100644
--- a/kernel/term.ml
+++ b/kernel/term.ml
@@ -271,7 +271,7 @@ let mkLambda (x,t1,t2) = IsLambda (x,t1,t2)
let mkLetIn (x,c1,t,c2) = IsLetIn (x,c1,t,c2)
(* If lt = [t1; ...; tn], constructs the application (t1 ... tn) *)
-(* We ensure applicative terms have at most one arguments and the
+(* We ensure applicative terms have at least one argument and the
function is not itself an applicative term *)
let mkApp (f, a) =
if a=[||] then f else
@@ -304,7 +304,6 @@ let mkFix fix = IsFix fix
let mkCoFix cofix = IsCoFix cofix
let kind_of_term c = c
-let mk_constr c = c
(*
end
diff --git a/kernel/term.mli b/kernel/term.mli
index fe8a888a6d..c8f6ea4a14 100644
--- a/kernel/term.mli
+++ b/kernel/term.mli
@@ -133,7 +133,6 @@ type cofixpoint = int * rec_declaration
term *)
val kind_of_term : constr -> (constr, types) kind_of_term
-val mk_constr : (constr, types) kind_of_term -> constr
(*s Term constructors. *)