aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded/Lexicographic_Exponentiation.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Wellfounded/Lexicographic_Exponentiation.v')
-rw-r--r--theories/Wellfounded/Lexicographic_Exponentiation.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v
index 24f5d308a..28288c0cb 100644
--- a/theories/Wellfounded/Lexicographic_Exponentiation.v
+++ b/theories/Wellfounded/Lexicographic_Exponentiation.v
@@ -130,7 +130,7 @@ Section Wf_Lexicographic_Exponentiation.
match goal with [ |- clos_refl_trans ?A ?R ?x ?y ] => cut (clos_refl A R x y) end.
intros; inversion H8; subst; [apply rt_step|apply rt_refl]; assumption.
generalize H1.
- rewrite H4; intro.
+ setoid_rewrite H4; intro.
generalize (app_inj_tail _ _ _ _ H8); simple induction 1.
intros.
@@ -182,7 +182,8 @@ Section Wf_Lexicographic_Exponentiation.
Descl x0 /\ Descl y0).
intro.
- generalize (app_nil_end x1); simple induction 1; simple induction 1.
+ generalize (app_nil_end x1).
+ simple induction 1; simple induction 1.
split. apply d_conc; auto with sets.
apply d_nil.