From a38d0b898b0d4e4c6535c4f583b4e3a56b3199b3 Mon Sep 17 00:00:00 2001 From: herbelin Date: Sun, 28 Mar 2004 14:41:46 +0000 Subject: Passage a un 'if-then-else' ou ne sont mentionnes que les membres droits qui sont supposes sans dependances en les arguments des constructeurs git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5589 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Bool/DecBool.v | 2 +- theories/Lists/TheoryList.v | 2 +- 2 files changed, 2 insertions(+), 2 deletions(-) (limited to 'theories') diff --git a/theories/Bool/DecBool.v b/theories/Bool/DecBool.v index 8a15e7624..2a0b2063d 100755 --- a/theories/Bool/DecBool.v +++ b/theories/Bool/DecBool.v @@ -11,7 +11,7 @@ Set Implicit Arguments. Definition ifdec (A B:Prop) (C:Set) (H:{A} + {B}) (x y:C) : C := - if H then fun _ => x else fun _ => y. + if H then x else y. Theorem ifdec_left : diff --git a/theories/Lists/TheoryList.v b/theories/Lists/TheoryList.v index 20f39e0ef..7671b25ff 100755 --- a/theories/Lists/TheoryList.v +++ b/theories/Lists/TheoryList.v @@ -149,7 +149,7 @@ Hypothesis eqA_dec : forall a b:A, {a = b} + {a <> b}. Fixpoint mem (a:A) (l:list A) {struct l} : bool := match l with | nil => false - | b :: m => if eqA_dec a b then fun H => true else fun H => mem a m + | b :: m => if eqA_dec a b then true else mem a m end. Hint Unfold In. -- cgit v1.2.3