aboutsummaryrefslogtreecommitdiff
path: root/lib
diff options
context:
space:
mode:
authorletouzey2012-10-02 15:58:00 +0000
committerletouzey2012-10-02 15:58:00 +0000
commit85c509a0fada387d3af96add3dac6a7c702b5d01 (patch)
tree4d262455aed52c20af0a9627d47d29b03ca6523d /lib
parent3415801b2c368ce03f6e8d33a930b9ab9e0b9fd1 (diff)
Remove some more "open" and dead code thanks to OCaml4 warnings
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15844 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'lib')
-rw-r--r--lib/cList.ml12
-rw-r--r--lib/dyn.ml1
-rw-r--r--lib/gmapl.ml1
-rw-r--r--lib/serialize.ml5
-rw-r--r--lib/store.ml10
-rw-r--r--lib/system.ml2
-rw-r--r--lib/util.ml5
-rw-r--r--lib/xml_parser.ml1
8 files changed, 0 insertions, 37 deletions
diff --git a/lib/cList.ml b/lib/cList.ml
index 2bf8d3597b..62d1ec3c14 100644
--- a/lib/cList.ml
+++ b/lib/cList.ml
@@ -550,13 +550,6 @@ let rec sep_last = function
| hd::[] -> (hd,[])
| hd::tl -> let (l,tl) = sep_last tl in (l,hd::tl)
-let try_find_i f =
- let rec try_find_f n = function
- | [] -> failwith "try_find_i"
- | h::t -> try f n h with Failure _ -> try_find_f (n+1) t
- in
- try_find_f
-
let rec find_map f = function
| [] -> raise Not_found
| x :: l ->
@@ -670,11 +663,6 @@ let rec split3 = function
| (x,y,z)::l ->
let (rx, ry, rz) = split3 l in (x::rx, y::ry, z::rz)
-let rec insert_in_class f a = function
- | [] -> [[a]]
- | (b::_ as l)::classes when f a b -> (a::l)::classes
- | l::classes -> l :: insert_in_class f a classes
-
let firstn n l =
let rec aux acc = function
| (0, l) -> List.rev acc
diff --git a/lib/dyn.ml b/lib/dyn.ml
index 13d1ec0608..de5158b141 100644
--- a/lib/dyn.ml
+++ b/lib/dyn.ml
@@ -7,7 +7,6 @@
(************************************************************************)
open Errors
-open Util
(* Dynamics, programmed with DANGER !!! *)
diff --git a/lib/gmapl.ml b/lib/gmapl.ml
index 5e8f27dc79..4be8f4baf6 100644
--- a/lib/gmapl.ml
+++ b/lib/gmapl.ml
@@ -6,7 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Errors
open Util
type ('a,'b) t = ('a,'b list) Gmap.t
diff --git a/lib/serialize.ml b/lib/serialize.ml
index 3ad508d74c..76a8b2c060 100644
--- a/lib/serialize.ml
+++ b/lib/serialize.ml
@@ -67,7 +67,6 @@ let goals : goals option call = Goal
let evars : evar list option call = Evars
let hints : (hint list * hint) option call = Hints
let status : status call = Status
-let search flags : string coq_object list call = Search flags
let get_options : (option_name * option_state) list call = GetOptions
let set_options l : unit call = SetOptions l
let inloadpath s : bool call = InLoadPath s
@@ -125,10 +124,6 @@ let do_match constr t mf = match constr with
else raise Marshal_error
| _ -> raise Marshal_error
-let pcdata = function
-| PCData s -> s
-| _ -> raise Marshal_error
-
let singleton = function
| [x] -> x
| _ -> raise Marshal_error
diff --git a/lib/store.ml b/lib/store.ml
index bc1b335fd0..ad6595adec 100644
--- a/lib/store.ml
+++ b/lib/store.ml
@@ -11,16 +11,6 @@
(* We give a short implementation of a universal type. This is mostly equivalent
to what is proposed by module Dyn.ml, except that it requires no explicit tag. *)
-module type Universal = sig
- type t
-
- type 'a etype = {
- put : 'a -> t ;
- get : t -> 'a option
- }
-
- val embed : unit -> 'a etype
-end
(* We use a dynamic "name" allocator. But if we needed to serialise stores, we
might want something static to avoid troubles with plugins order. *)
diff --git a/lib/system.ml b/lib/system.ml
index cf650d6abc..6076217b30 100644
--- a/lib/system.ml
+++ b/lib/system.ml
@@ -92,8 +92,6 @@ let is_in_path lpath filename =
try ignore (where_in_path ~warn:false lpath filename); true
with Not_found -> false
-let path_separator = if Sys.os_type = "Unix" then ':' else ';'
-
let is_in_system_path filename =
let path = try Sys.getenv "PATH"
with Not_found -> error "system variable PATH not found" in
diff --git a/lib/util.ml b/lib/util.ml
index 6240759566..af3b13fa7d 100644
--- a/lib/util.ml
+++ b/lib/util.ml
@@ -24,11 +24,6 @@ let pi1 (a,_,_) = a
let pi2 (_,a,_) = a
let pi3 (_,_,a) = a
-(* Projection operator *)
-
-let down_fst f x = f (fst x)
-let down_snd f x = f (snd x)
-
(* Characters *)
let is_letter c = (c >= 'a' && c <= 'z') or (c >= 'A' && c <= 'Z')
diff --git a/lib/xml_parser.ml b/lib/xml_parser.ml
index 6207763cda..783f5c91b6 100644
--- a/lib/xml_parser.ml
+++ b/lib/xml_parser.ml
@@ -98,7 +98,6 @@ let make source =
}
let check_eof p v = p.check_eof <- v
-let concat_pcdata p v = p.concat_pcdata <- v
let pop s =
try