From ca43236e7c78090f103c7b5716bd89d796416d87 Mon Sep 17 00:00:00 2001 From: herbelin Date: Wed, 16 Nov 2011 08:46:35 +0000 Subject: Suppression fichier Case8.v redondant git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14658 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/ideal-features/Case8.v | 36 ------------------------------------ 1 file changed, 36 deletions(-) delete mode 100644 test-suite/ideal-features/Case8.v (limited to 'test-suite/ideal-features') diff --git a/test-suite/ideal-features/Case8.v b/test-suite/ideal-features/Case8.v deleted file mode 100644 index 2ac5bd8c0..000000000 --- a/test-suite/ideal-features/Case8.v +++ /dev/null @@ -1,36 +0,0 @@ -Inductive listn : nat -> Set := - | niln : listn 0 - | consn : forall n : nat, nat -> listn n -> listn (S n). - -Inductive empty : forall n : nat, listn n -> Prop := - intro_empty : empty 0 niln. - -Parameter - inv_empty : forall (n a : nat) (l : listn n), ~ empty (S n) (consn n a l). - -Type - (fun (n : nat) (l : listn n) => - match l in (listn n) return (empty n l \/ ~ empty n l) with - | niln => or_introl (~ empty 0 niln) intro_empty - | consn n O y as b => or_intror (empty (S n) b) (inv_empty n 0 y) - | consn n a y as b => or_intror (empty (S n) b) (inv_empty n a y) - end). - - -Type - (fun (n : nat) (l : listn n) => - match l in (listn n) return (empty n l \/ ~ empty n l) with - | niln => or_introl (~ empty 0 niln) intro_empty - | consn n O y => or_intror (empty (S n) (consn n 0 y)) (inv_empty n 0 y) - | consn n a y => or_intror (empty (S n) (consn n a y)) (inv_empty n a y) - end). - - - -Type - (fun (n : nat) (l : listn n) => - match l in (listn n) return (empty n l \/ ~ empty n l) with - | niln => or_introl (~ empty 0 niln) intro_empty - | consn O a y as b => or_intror (empty 1 b) (inv_empty 0 a y) - | consn n a y as b => or_intror (empty (S n) b) (inv_empty n a y) - end). -- cgit v1.2.3