aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/correctness/pmisc.ml
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-04 14:13:24 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-04 14:13:24 +0000
commit0df14c3d0d2c71716bbed04451ad2e2541dcc6a3 (patch)
treeec4918a0ef86b133860847f1b61e858b0920d6a1 /contrib/correctness/pmisc.ml
parent2def0e4f8e5d075d815df253d316a96dd7257423 (diff)
renommage du module Pcoq.Vernac en Pcoq.Vernac_ pour contourner un bug d'ocamldep
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1547 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/correctness/pmisc.ml')
-rw-r--r--contrib/correctness/pmisc.ml18
1 files changed, 9 insertions, 9 deletions
diff --git a/contrib/correctness/pmisc.ml b/contrib/correctness/pmisc.ml
index f25541961..77356e17c 100644
--- a/contrib/correctness/pmisc.ml
+++ b/contrib/correctness/pmisc.ml
@@ -17,6 +17,8 @@ open Term
module SpSet = Set.Make(struct type t = section_path let compare = sp_ord end)
+let coq_constant d s = make_path ("Coq" :: d) (id_of_string s) CCI
+
(* debug *)
let debug = ref false
@@ -159,22 +161,20 @@ let is_connective id =
(* [conj i s] constructs the conjunction of two constr *)
-let conj i s =
- Term.applist (constant "and", [i; s])
-
+let conj i s = Term.applist (constant "and", [i; s])
-(* [n_mkNamedProd v [xn,tn;...;x1,t1]] constructs the type (x1:t1)...(xn:tn)v
- *)
+(* [n_mkNamedProd v [xn,tn;...;x1,t1]] constructs the type
+ [(x1:t1)...(xn:tn)v] *)
let rec n_mkNamedProd v = function
- [] -> v
- | (id,ty)::rem -> n_mkNamedProd (Term.mkNamedProd id ty v) rem
+ | [] -> v
+ | (id,ty) :: rem -> n_mkNamedProd (Term.mkNamedProd id ty v) rem
(* [n_lambda v [xn,tn;...;x1,t1]] constructs the type [x1:t1]...[xn:tn]v *)
let rec n_lambda v = function
- [] -> v
- | (id,ty)::rem -> n_lambda (Term.mkNamedLambda id ty v) rem
+ | [] -> v
+ | (id,ty) :: rem -> n_lambda (Term.mkNamedLambda id ty v) rem
(* [abstract env idl c] constructs [x1]...[xn]c where idl = [x1;...;xn] *)