aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-06-29 10:50:27 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-06-29 10:50:27 +0000
commiteee66457ddfd86c65cc1287b4545f828bf43f2dd (patch)
tree6de3973e9c383942f47a372c20614454bcf43e3d
parent124f43b6666a2aca97a3189f970dd76e0851c178 (diff)
Rien
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@522 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--proofs/logic.ml2
-rw-r--r--proofs/pattern.ml2
-rw-r--r--tactics/tactics.ml2
3 files changed, 3 insertions, 3 deletions
diff --git a/proofs/logic.ml b/proofs/logic.ml
index 2f59990d6..5f8d7c2f2 100644
--- a/proofs/logic.ml
+++ b/proofs/logic.ml
@@ -136,7 +136,7 @@ varaibles only in Application and Case *)
let collect_meta_variables c =
let rec collrec acc = function
| DOP0(Meta mv) -> mv::acc
- | DOP2(Cast,c,t) -> collrec acc c
+ | DOP2(Cast,c,_) -> collrec acc c
| DOPN(AppL,cl) -> Array.fold_left collrec acc cl
| DOPN(MutCase _,_) as mc ->
let (_,p,c,lf) = destCase mc in
diff --git a/proofs/pattern.ml b/proofs/pattern.ml
index 983154c80..6d3c362d6 100644
--- a/proofs/pattern.ml
+++ b/proofs/pattern.ml
@@ -221,7 +221,7 @@ let rec pattern_of_constr t =
| IsVar id -> PRef (RVar id)
| IsSort (Prop c) -> PSort (RProp c)
| IsSort (Type _) -> PSort RType
- | IsCast (c,t) -> pattern_of_constr c
+ | IsCast (c,_) -> pattern_of_constr c
| IsProd (na,c,b) ->
PBinder (BProd,na,pattern_of_constr c,pattern_of_constr b)
| IsLambda (na,c,b) ->
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index feb4bf69a..9a03eca97 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -1038,7 +1038,7 @@ let induct_discharge indpath statuslists cname destopt avoid (_,t) =
[ central_intro (IBasedOn (recvarname,avoid)) destopt false;
central_intro (IBasedOn (hyprecname,avoid)) None false;
peel_tac c]
- | DOP2 (Cast,c,t) -> peel_tac c
+ | DOP2 (Cast,c,_) -> peel_tac c
| DOP2 (Prod,t,DLAM(na,c))
-> tclTHEN (central_intro (IAvoid avoid) destopt false)
(peel_tac c)