aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapFullAVL.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/FSets/FMapFullAVL.v')
-rw-r--r--theories/FSets/FMapFullAVL.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/FSets/FMapFullAVL.v b/theories/FSets/FMapFullAVL.v
index 59b778369..dea23d68c 100644
--- a/theories/FSets/FMapFullAVL.v
+++ b/theories/FSets/FMapFullAVL.v
@@ -726,7 +726,7 @@ Module IntMake_ord (I:Int)(X: OrderedType)(D : OrderedType) <:
intros.
assert (H1:=cons_1 m1 (Raw.End _)).
assert (H2:=cons_1 m2 (Raw.End _)).
- simpl in *; rewrite <- app_nil_end in *; rewrite <-H1,<-H2.
+ simpl in *; rewrite app_nil_r in *; rewrite <-H1,<-H2.
apply (@compare_aux_Cmp (Raw.cons m1 (Raw.End _),
Raw.cons m2 (Raw.End _))).
Qed.