From 183112fc6a5fbb7d1c6d60b9717cdb8aceda78ca Mon Sep 17 00:00:00 2001 From: Pierre Boutillier Date: Mon, 8 Sep 2014 16:19:39 +0200 Subject: Simpl less (so that cbn will not simpl too much) --- plugins/btauto/Reflect.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) (limited to 'plugins/btauto/Reflect.v') 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. -- cgit v1.2.3