aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/mltop.ml
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-12 18:52:09 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-12 18:52:09 +0100
commitde8888e28ad793511ba2e2969516325b0be44330 (patch)
treef910699eb3afb1f2b1835a01e8529c48c950b861 /toplevel/mltop.ml
parent9daec838c8896e7c1048b42d01eba0c71c912f00 (diff)
Revert "Using same code for browsing physical directories in coqtop and coqdep."
(Sorry, was not intended to be pushed) This reverts commit 5268efdefb396267bfda0c17eb045fa2ed516b3c.
Diffstat (limited to 'toplevel/mltop.ml')
-rw-r--r--toplevel/mltop.ml3
1 files changed, 1 insertions, 2 deletions
diff --git a/toplevel/mltop.ml b/toplevel/mltop.ml
index ef2e62c3b..357c5482f 100644
--- a/toplevel/mltop.ml
+++ b/toplevel/mltop.ml
@@ -11,7 +11,6 @@ open Util
open Pp
open Flags
open Libobject
-open Systemdirs
open System
(* Code to hook Coq into the ML toplevel -- depends on having the
@@ -156,7 +155,7 @@ let add_ml_dir s =
| WithoutTop when has_dynlink -> keep_copy_mlpath s
| _ -> ()
-(* For Rec Add ML Path (-R) *)
+(* For Rec Add ML Path *)
let add_rec_ml_dir unix_path =
List.iter (fun (lp,_) -> add_ml_dir lp) (all_subdirs ~unix_path)