aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-04 17:09:57 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-04 17:09:57 +0000
commit885673cbec549d24bd57b9e16bfb5375e426101c (patch)
treec3693a4e70758d70e9706f7f98c54f6f1bfa0ab7 /toplevel
parentcc92b9228f3463ce06ad457a47ef2a9b1f39a727 (diff)
Modification Require From
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3376 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/vernacentries.ml6
-rw-r--r--toplevel/vernacexpr.ml2
2 files changed, 4 insertions, 4 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 9b977b846..c911633e8 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -558,8 +558,8 @@ let vernac_solve_existential = instantiate_nth_evar_com
(*****************************)
(* Auxiliary file management *)
-let vernac_require_from export spec id filename =
- Library.require_library_from_file spec (Some id) filename export
+let vernac_require_from export spec filename =
+ Library.require_library_from_file spec None filename export
let vernac_add_loadpath isrec pdir ldiropt =
let alias = match ldiropt with
@@ -1077,7 +1077,7 @@ let interp c = match c with
| VernacSolveExistential (n,c) -> vernac_solve_existential n c
(* Auxiliary file and library management *)
- | VernacRequireFrom (exp,spec,id,f) -> vernac_require_from exp spec id f
+ | VernacRequireFrom (exp,spec,f) -> vernac_require_from exp spec f
| VernacAddLoadPath (isrec,s,alias) -> vernac_add_loadpath isrec s alias
| VernacRemoveLoadPath s -> vernac_remove_loadpath s
| VernacAddMLPath (isrec,s) -> vernac_add_ml_path isrec s
diff --git a/toplevel/vernacexpr.ml b/toplevel/vernacexpr.ml
index 36c277b95..a11eadc7e 100644
--- a/toplevel/vernacexpr.ml
+++ b/toplevel/vernacexpr.ml
@@ -203,7 +203,7 @@ type vernac_expr =
| VernacSolveExistential of int * constr_expr
(* Auxiliary file and library management *)
- | VernacRequireFrom of export_flag * specif_flag option * identifier * string
+ | VernacRequireFrom of export_flag * specif_flag option * string
| VernacAddLoadPath of rec_flag * string * dir_path option
| VernacRemoveLoadPath of string
| VernacAddMLPath of rec_flag * string