aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/rtauto
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-12-28 16:26:45 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-12-28 16:26:45 +0000
commit380acdd0100d55cd908a96731365c1ce287e2d10 (patch)
tree7fa607978bfb166517a19e3e464de2544063e5fb /contrib/rtauto
parentd556fd3ffb8b59e2a5136ab748a3a8d73c3f45f0 (diff)
Remplacement de la définition de Pind et Prec par une définition
suggérée par Conor McBride qui ne fait pas intervenir eq_rect et qui permet de montrer "facilement" (mais avec l'axiome K) les équations de réduction de Prec. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9465 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/rtauto')
-rw-r--r--contrib/rtauto/Bintree.v9
1 files changed, 0 insertions, 9 deletions
diff --git a/contrib/rtauto/Bintree.v b/contrib/rtauto/Bintree.v
index 8827da100..67a952b73 100644
--- a/contrib/rtauto/Bintree.v
+++ b/contrib/rtauto/Bintree.v
@@ -20,15 +20,6 @@ Ltac caseq t := generalize (refl_equal t); pattern t at -1; case t.
Functional Scheme Pcompare_ind := Induction for Pcompare Sort Prop.
-Lemma Prect : forall P : positive -> Type,
- P 1 ->
- (forall n : positive, P n -> P (Psucc n)) -> forall p : positive, P p.
-intros P H1 Hsucc n; induction n.
-rewrite <- plus_iter_xI; apply Hsucc; apply iterate_add; assumption.
-rewrite <- plus_iter_xO; apply iterate_add; assumption.
-assumption.
-Qed.
-
Lemma Gt_Eq_Gt : forall p q cmp,
(p ?= q) Eq = Gt -> (p ?= q) cmp = Gt.
apply (Pcompare_ind (fun p q cmp _ => (p ?= q) Eq = Gt -> (p ?= q) cmp = Gt));