aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/btauto
diff options
context:
space:
mode:
authorGravatar Pierre Boutillier <pierre.boutillier@pps.univ-paris-diderot.fr>2014-09-08 16:19:39 +0200
committerGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-10-01 23:24:36 +0200
commit183112fc6a5fbb7d1c6d60b9717cdb8aceda78ca (patch)
tree8ac0350e08c22893acbb3905e028aee18f86bb5b /plugins/btauto
parentb9a6247ddc52082065b56f296c889c41167e0507 (diff)
Simpl less (so that cbn will not simpl too much)
Diffstat (limited to 'plugins/btauto')
-rw-r--r--plugins/btauto/Reflect.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/plugins/btauto/Reflect.v b/plugins/btauto/Reflect.v
index 8a95d5b4b..3bd7cd622 100644
--- a/plugins/btauto/Reflect.v
+++ b/plugins/btauto/Reflect.v
@@ -196,9 +196,9 @@ Qed.
Lemma make_last_nth_1 : forall A n i x def, i <> n ->
list_nth i (@make_last A n x def) def = def.
Proof.
-intros A n; induction n using Pos.peano_rect; intros i x def Hd; simpl.
-+ unfold make_last; rewrite Pos.peano_rect_base.
- induction i using Pos.peano_case; [elim Hd; reflexivity|].
+intros A n; induction n using Pos.peano_rect; intros i x def Hd;
+ unfold make_last; simpl.
++ induction i using Pos.peano_case; [elim Hd; reflexivity|].
rewrite list_nth_succ, list_nth_nil; reflexivity.
+ unfold make_last; rewrite Pos.peano_rect_succ; fold (make_last n x def).
induction i using Pos.peano_case.