aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/CasesDep.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-02 16:23:10 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-02 16:23:10 +0000
commit6e2ca58652b23415cba082c4be77823f182d14ba (patch)
tree633f10ce82f08cd830d2216db05f6b672a204b08 /test-suite/success/CasesDep.v
parent46cad49197abd858ef430c150e32702c01b2f205 (diff)
Minor fixes. Use expanded type in class_tactics for Morphism search, to
alleviate some problems with delta. Better precedence in lambda notation. Temporarily deactivate notations for relation conjunction, equivalence and so on, while we search for a better syntax and maybe a generalization (fixes bug #1820). Better destruct_call in Program.Tactics. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10742 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/CasesDep.v')
-rw-r--r--test-suite/success/CasesDep.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/CasesDep.v b/test-suite/success/CasesDep.v
index 0d71df82f..b625eb151 100644
--- a/test-suite/success/CasesDep.v
+++ b/test-suite/success/CasesDep.v
@@ -478,3 +478,9 @@ match l return l = l with
end
| _ => refl_equal _
end.
+
+Fixpoint app {A} {n m} (v : listn A n) (w : listn A m) : listn A (n + m) :=
+ match v with
+ | niln => w
+ | consn a n' v' => consn _ a _ (app v' w)
+ end.