aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-20 19:46:21 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-12-20 19:46:21 +0000
commitb9da9226ebd8a2db21570ba269663e16f63e1815 (patch)
tree0edbf36cc7ad7804833bb607801b525a3dac57ce /theories
parent296fb02406b92203339e6493ede9b9ef0d65075b (diff)
Rétablissement de l'ancien comportement de Simpl sauf dans le cas mutuel inductif où la constante la plus proche du Fix est prise en compte
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1169 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Arith/Div2.v7
-rw-r--r--theories/Zarith/auxiliary.v2
2 files changed, 8 insertions, 1 deletions
diff --git a/theories/Arith/Div2.v b/theories/Arith/Div2.v
index a2187a89b..202e7a97a 100644
--- a/theories/Arith/Div2.v
+++ b/theories/Arith/Div2.v
@@ -113,11 +113,18 @@ Intros. Decompose [and] H. Unfold iff in H0 H1.
Decompose [and] H0. Decompose [and] H1. Clear H H0 H1.
Split; Split.
Intro H. Inversion H. Inversion H1.
+Simpl. Rewrite (double_S (div2 n0)). Auto with arith.
+Simpl. Rewrite (double_S (div2 n0)). Intro H. Injection H. Auto with arith.
+Intro H. Inversion H. Inversion H1.
+Simpl. Rewrite (double_S (div2 n0)). Auto with arith.
+Simpl. Rewrite (double_S (div2 n0)). Intro H. Injection H. Auto with arith.
+(*
Simpl. Rewrite <- plus_n_Sm. Auto with arith.
Simpl. Rewrite <- plus_n_Sm. Intro H. Injection H. Auto with arith.
Intro H. Inversion H. Inversion H1.
Simpl. Rewrite <- plus_n_Sm. Auto with arith.
Simpl. Rewrite <- plus_n_Sm. Intro H. Injection H. Auto with arith.
+*)
Qed.
diff --git a/theories/Zarith/auxiliary.v b/theories/Zarith/auxiliary.v
index 0f0fbc52b..e7bcdcfab 100644
--- a/theories/Zarith/auxiliary.v
+++ b/theories/Zarith/auxiliary.v
@@ -388,7 +388,7 @@ Save.
Lemma add_x_x : (x:positive) (add x x) = (xO x).
Intros p; Apply convert_intro; Simpl; Rewrite convert_add;
-Rewrite ZL6; Trivial with arith.
+Unfold 3 convert ; Simpl; Rewrite ZL6; Trivial with arith.
Save.
Theorem Zcompare_Zmult_compatible :