aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-22 14:35:51 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-22 14:35:51 +0000
commitd619a834de7548649f53d59ec4fc9e892b33d24c (patch)
tree10bb2d3e30caeccfada2e2d812a56cf416e8d89a /theories
parent2debc4ab0b171963afff40cc3183e4e92cca9a0e (diff)
A try at allowing matching on applications as a binary syntax node by default.
It breaks tauto as [?X _ _] matches much more terms. It is mostly fixed by not destructing objects of record types. The new [intuition] was also pulling an unneeded dependency in Field_theory which can be cleared easily. Zis_gcd_bezout is also considered a conjunction now, which seems correct(?). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11243 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/QArith/Qreduction.v4
-rw-r--r--theories/ZArith/Znumtheory.v5
2 files changed, 5 insertions, 4 deletions
diff --git a/theories/QArith/Qreduction.v b/theories/QArith/Qreduction.v
index 6b16cfff4..f289b6106 100644
--- a/theories/QArith/Qreduction.v
+++ b/theories/QArith/Qreduction.v
@@ -49,7 +49,7 @@ Proof.
Open Scope Z_scope.
intuition.
rewrite <- H in H0,H1; clear H.
- rewrite H3; rewrite H4.
+ rewrite H5; rewrite H6.
assert (0 <> g).
intro; subst g; discriminate.
@@ -57,7 +57,7 @@ Proof.
apply Zmult_gt_0_lt_0_reg_r with g.
omega.
rewrite Zmult_comm.
- rewrite <- H4; compute; auto.
+ rewrite <- H6; compute; auto.
rewrite Z2P_correct; auto.
ring.
Close Scope Z_scope.
diff --git a/theories/ZArith/Znumtheory.v b/theories/ZArith/Znumtheory.v
index cbe65989e..599d6791a 100644
--- a/theories/ZArith/Znumtheory.v
+++ b/theories/ZArith/Znumtheory.v
@@ -521,8 +521,9 @@ Qed.
Lemma Zis_gcd_mult :
forall a b c d:Z, Zis_gcd a b d -> Zis_gcd (c * a) (c * b) (c * d).
Proof.
- intros a b c d; simple induction 1; constructor; intuition.
- elim (Zis_gcd_bezout a b d H); intros.
+ intros a b c d; simple induction 1; constructor.
+ intuition. intuition. intros. intuition.
+ elim (Zis_gcd_bezout a b d H). intros.
elim H3; intros.
elim H4; intros.
apply Zdivide_intro with (u * q + v * q0).