From d90205f6284b998a8fc50b295d2d790d2580ea26 Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Fri, 11 Jul 2014 19:30:08 +0200 Subject: Fix Funind test-suite file after patch by Pierre. --- test-suite/success/Funind.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) diff --git a/test-suite/success/Funind.v b/test-suite/success/Funind.v index dcf7b249a..3bf97c131 100644 --- a/test-suite/success/Funind.v +++ b/test-suite/success/Funind.v @@ -151,7 +151,7 @@ Function nat_equal_bool (n m : nat) {struct n} : bool := Require Export Div2. - +Require Import Nat. Functional Scheme div2_ind := Induction for div2 Sort Prop. Lemma div2_inf : forall n : nat, div2 n <= n. intros n. @@ -234,11 +234,11 @@ Qed. Inductive istrue : bool -> Prop := istrue0 : istrue true. -Functional Scheme plus_ind := Induction for plus Sort Prop. +Functional Scheme add_ind := Induction for add Sort Prop. Lemma inf_x_plusxy' : forall x y : nat, x <= x + y. intros n m. - functional induction plus n m; intros. + functional induction add n m; intros. auto with arith. auto with arith. Qed. -- cgit v1.2.3