diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2004-03-11 23:40:36 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2004-03-11 23:40:36 +0000 |
commit | 3320a366786ef02842b1327ebace1a1203b1e1b6 (patch) | |
tree | f5d64f49aaded015c540e7b290cc43e2e65b8be1 /test-suite | |
parent | 194902c54308e83aba33852eee69e3370879972c (diff) |
Ajout exemple Inst
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5459 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/success/ltac.v | 13 |
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/success/ltac.v b/test-suite/success/ltac.v index 880f92fdd..55aa110d2 100644 --- a/test-suite/success/ltac.v +++ b/test-suite/success/ltac.v @@ -55,3 +55,16 @@ Qed. Lemma back3 : (0)=(0)->(1)=(1)->(0)=(1)->(0)=(0). Intros; Match Context With [_:(O)=?1;_:(1)=(1)|-? ] -> Exact (refl_equal ? ?1). Qed. + +(* Check context binding *) +Tactic Definition sym t := Match t With [C[?1=?2]] -> Inst C[?1=?2]. + +Lemma sym : ~(0)=(1)->~(1)=(0). +Intro H. +Let t = (sym (Check H)) In Assert t. +Exact H. +Intro H1. +Apply H. +Symmetry. +Assumption. +Qed. |