aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/dependentind.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-03 14:41:08 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-03 14:41:08 +0000
commit6832c60f741e6bfb2a850d567fd6a1dff7059393 (patch)
treea31e0d9937437aa884c611a8554b80baaeae0811 /test-suite/success/dependentind.v
parentb467ab92ef5bd124ae2bd19deea58765bd034f83 (diff)
Minor fixes related to coqdoc and --interpolate and the dependent
induction test-suite script. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11426 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/dependentind.v')
-rw-r--r--test-suite/success/dependentind.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/test-suite/success/dependentind.v b/test-suite/success/dependentind.v
index 3f315ccb7..d12c21b15 100644
--- a/test-suite/success/dependentind.v
+++ b/test-suite/success/dependentind.v
@@ -58,11 +58,13 @@ Inductive term : ctx -> type -> Type :=
Hint Constructors term : lambda.
+Open Local Scope context_scope.
+
Notation " Γ |-- τ " := (term Γ τ) (at level 0) : type_scope.
Lemma weakening : forall Γ Δ τ, term (Γ ;; Δ) τ ->
forall τ', term (Γ ,, τ' ;; Δ) τ.
-Proof with simpl in * ; simplify_dep_elim ; simplify_IH_hyps ; eauto with lambda.
+Proof with simpl in * ; reverse ; simplify_dep_elim ; simplify_IH_hyps ; eauto with lambda.
intros Γ Δ τ H.
dependent induction H.
@@ -81,7 +83,7 @@ Proof with simpl in * ; simplify_dep_elim ; simplify_IH_hyps ; eauto with lambda
Qed.
Lemma exchange : forall Γ Δ α β τ, term (Γ,, α,, β ;; Δ) τ -> term (Γ,, β,, α ;; Δ) τ.
-Proof with simpl in * ; simplify_dep_elim ; simplify_IH_hyps ; auto.
+Proof with simpl in * ; subst ; reverse ; simplify_dep_elim ; simplify_IH_hyps ; auto.
intros until 1.
dependent induction H.