summaryrefslogtreecommitdiff
path: root/test-suite/success/fix.v
diff options
context:
space:
mode:
authorGravatar Stephane Glondu <steph@glondu.net>2013-05-08 18:01:07 +0200
committerGravatar Stephane Glondu <steph@glondu.net>2013-05-08 18:01:07 +0200
commit095eac936751bab72e3c6bbdfa3ede51f7198721 (patch)
tree44cf2859ba6b8486f056efaaf7ee6c2d855f2aae /test-suite/success/fix.v
parent4e6d6dab2ef2de6c1ad7972fc981e55a4fde7ae3 (diff)
parent0b14713e3efd7f8f1cc8a06555d0ec8fbe496130 (diff)
Merge branch 'experimental/master'
Diffstat (limited to 'test-suite/success/fix.v')
-rw-r--r--test-suite/success/fix.v9
1 files changed, 4 insertions, 5 deletions
diff --git a/test-suite/success/fix.v b/test-suite/success/fix.v
index be4e0684..8623f718 100644
--- a/test-suite/success/fix.v
+++ b/test-suite/success/fix.v
@@ -9,17 +9,16 @@ Inductive rBoolOp : Set :=
| rAnd : rBoolOp
| rEq : rBoolOp.
-Definition rlt (a b : rNat) : Prop :=
- (a ?= b)%positive Datatypes.Eq = Datatypes.Lt.
+Definition rlt (a b : rNat) : Prop := Pos.compare_cont a b Eq = Lt.
Definition rltDec : forall m n : rNat, {rlt m n} + {rlt n m \/ m = n}.
intros n m; generalize (nat_of_P_lt_Lt_compare_morphism n m);
generalize (nat_of_P_gt_Gt_compare_morphism n m);
- generalize (Pcompare_Eq_eq n m); case ((n ?= m)%positive Datatypes.Eq).
+ generalize (Pcompare_Eq_eq n m); case (Pos.compare_cont n m Eq).
intros H' H'0 H'1; right; right; auto.
-intros H' H'0 H'1; left; unfold rlt in |- *.
+intros H' H'0 H'1; left; unfold rlt.
apply nat_of_P_lt_Lt_compare_complement_morphism; auto.
-intros H' H'0 H'1; right; left; unfold rlt in |- *.
+intros H' H'0 H'1; right; left; unfold rlt.
apply nat_of_P_lt_Lt_compare_complement_morphism; auto.
apply H'0; auto.
Defined.