From 5b7eafd0f00a16d78f99a27f5c7d5a0de77dc7e6 Mon Sep 17 00:00:00 2001 From: Stephane Glondu Date: Wed, 21 Jul 2010 09:46:51 +0200 Subject: Imported Upstream snapshot 8.3~beta0+13298 --- plugins/subtac/test/take.v | 34 ++++++++++++++++++++++++++++++++++ 1 file changed, 34 insertions(+) create mode 100644 plugins/subtac/test/take.v (limited to 'plugins/subtac/test/take.v') diff --git a/plugins/subtac/test/take.v b/plugins/subtac/test/take.v new file mode 100644 index 00000000..90ae8bae --- /dev/null +++ b/plugins/subtac/test/take.v @@ -0,0 +1,34 @@ +(* -*- coq-prog-args: ("-emacs-U" "-debug") -*- *) +Require Import JMeq. +Require Import List. +Require Import Program. + +Set Implicit Arguments. +Obligations Tactic := idtac. + +Print cons. + +Program Fixpoint take (A : Set) (l : list A) (n : nat | n <= length l) { struct l } : { l' : list A | length l' = n } := + match n with + | 0 => nil + | S p => + match l with + | cons hd tl => let rest := take tl p in cons hd rest + | nil => ! + end + end. + +Require Import Omega. +Solve All Obligations. +Next Obligation. + destruct_call take ; program_simpl. +Defined. + +Next Obligation. + intros. + inversion H. +Defined. + + + + -- cgit v1.2.3