aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-04-13 11:20:20 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-04-13 11:20:20 +0200
commit8b1b6e76a6229d9c091bf805e3786bdf0038ae32 (patch)
treef137e7b0f86a6f9a9df43cf8acaad573457e5205
parenta5c150a6a7fa980c5850aa247e62d02e29773235 (diff)
Silence a few OCaml warnings.
-rw-r--r--plugins/rtauto/refl_tauto.ml1
-rw-r--r--pretyping/patternops.ml2
-rw-r--r--stm/asyncTaskQueue.ml2
3 files changed, 2 insertions, 3 deletions
diff --git a/plugins/rtauto/refl_tauto.ml b/plugins/rtauto/refl_tauto.ml
index f30f8a943..3655df895 100644
--- a/plugins/rtauto/refl_tauto.ml
+++ b/plugins/rtauto/refl_tauto.ml
@@ -95,7 +95,6 @@ let rec make_form atom_env gls term =
let normalize=special_nf gls in
let cciterm=special_whd gls term in
let sigma = Tacmach.project gls in
- let inj = EConstr.Unsafe.to_constr in
match EConstr.kind sigma cciterm with
Prod(_,a,b) ->
if noccurn sigma 1 b &&
diff --git a/pretyping/patternops.ml b/pretyping/patternops.ml
index 318f94be2..2eff1936f 100644
--- a/pretyping/patternops.ml
+++ b/pretyping/patternops.ml
@@ -156,7 +156,7 @@ let pattern_of_constr env sigma t =
| Construct (sp,u) -> PRef (canonical_gr (ConstructRef sp))
| Proj (p, c) ->
pattern_of_constr env (EConstr.Unsafe.to_constr (Retyping.expand_projection env sigma p (EConstr.of_constr c) []))
- | Evar (evk,ctxt as ev) ->
+ | Evar (evk,ctxt) ->
(match snd (Evd.evar_source evk sigma) with
| Evar_kinds.MatchingVar (b,id) ->
assert (not b); PMeta (Some id)
diff --git a/stm/asyncTaskQueue.ml b/stm/asyncTaskQueue.ml
index 3459156a4..3fa1732a4 100644
--- a/stm/asyncTaskQueue.ml
+++ b/stm/asyncTaskQueue.ml
@@ -308,7 +308,7 @@ module Make(T : Task) = struct
(* We pass feedback to master *)
let slave_feeder oc fb =
Marshal.to_channel oc (RespFeedback (debug_with_pid fb)) []; flush oc in
- Feedback.add_feeder (fun x -> slave_feeder (Option.get !slave_oc) x);
+ ignore (Feedback.add_feeder (fun x -> slave_feeder (Option.get !slave_oc) x));
(* We ask master to allocate universe identifiers *)
Universes.set_remote_new_univ_level (bufferize (fun () ->
marshal_response (Option.get !slave_oc) RespGetCounterNewUnivLevel;