From 208a0f7bfa5249f9795e6e225f309cbe715c0fad Mon Sep 17 00:00:00 2001 From: Samuel Mimram Date: Tue, 21 Nov 2006 21:38:49 +0000 Subject: Imported Upstream version 8.1~gamma --- test-suite/success/Injection.v | 26 ++++++++++++++++++++++++++ 1 file changed, 26 insertions(+) (limited to 'test-suite/success/Injection.v') diff --git a/test-suite/success/Injection.v b/test-suite/success/Injection.v index f8f7c996..606e884a 100644 --- a/test-suite/success/Injection.v +++ b/test-suite/success/Injection.v @@ -36,3 +36,29 @@ intros. exact (fun H => H). Qed. +(* Test injection as *) + +Lemma l5 : forall x y z t : nat, (x,y) = (z,t) -> x=z. +intros; injection H as Hyt Hxz. +exact Hxz. +Qed. + +(* Injection does not projects at positions in Prop... allow it? + +Inductive t (A:Prop) : Set := c : A -> t A. +Goal forall p q : True\/True, c _ p = c _ q -> False. +intros. +injection H. +Abort. + +*) + +(* Accept does not project on discriminable positions... allow it? + +Goal 1=2 -> 1=0. +intro H. +injection H. +intro; assumption. +Qed. + + *) -- cgit v1.2.3