aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapList.v
diff options
context:
space:
mode:
authorGravatar jforest <jforest@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-06 11:09:43 +0000
committerGravatar jforest <jforest@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-06-06 11:09:43 +0000
commit923259f3cd17bccf2353b3734f8d9f5fb8d89351 (patch)
tree885cbccc36057bb171b036d2446c007c88513326 /theories/FSets/FMapList.v
parentc9f4643f733fbfa368cb4644f95b2e233d5ad973 (diff)
+ ameliorating the tactic "functional induction"
+ bug correction in proof of structural principles + up do to date test-suite/success/Funind.v git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8899 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapList.v')
-rw-r--r--theories/FSets/FMapList.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/theories/FSets/FMapList.v b/theories/FSets/FMapList.v
index 128ed45d2..5564b174b 100644
--- a/theories/FSets/FMapList.v
+++ b/theories/FSets/FMapList.v
@@ -112,7 +112,7 @@ Proof.
intros m Hm x; generalize Hm; clear Hm.
functional induction (mem x m);intros sorted belong1;trivial.
- inversion belong1. inversion H0.
+ inversion belong1. inversion H.
absurd (In x ((k', _x) :: l));try assumption.
apply Sort_Inf_NotIn with _x;auto.
@@ -200,7 +200,7 @@ Proof.
functional induction (add x e' m) ;simpl;auto; clear H0.
subst;auto.
- intros y' e'' eqky'; inversion_clear 1; destruct H1; simpl in *.
+ intros y' e'' eqky'; inversion_clear 1; destruct H0; simpl in *.
order.
auto.
auto.
@@ -213,10 +213,10 @@ Lemma add_3 : forall m x y e e',
Proof.
intros m x y e e'. generalize y e; clear y e; unfold PX.MapsTo.
functional induction (add x e' m);simpl; intros.
+ apply (In_inv_3 H0); compute; auto.
apply (In_inv_3 H1); compute; auto.
- subst s;apply (In_inv_3 H2); compute; auto.
- constructor 2; apply (In_inv_3 H2); compute; auto.
- inversion_clear H2; auto.
+ constructor 2; apply (In_inv_3 H1); compute; auto.
+ inversion_clear H1; auto.
Qed.
@@ -441,8 +441,8 @@ Proof.
apply Inf_lt with (x,e); auto.
elim (Sort_Inf_NotIn H5 H7 H4).
- destruct _x;
- destruct _x0;try contradiction.
+ destruct m;
+ destruct m';try contradiction.
clear H1;destruct p as (k,e).
destruct (H0 k).