From 9b9eb66140e67b4815bffc21984056516b10e111 Mon Sep 17 00:00:00 2001 From: glondu Date: Sun, 2 Nov 2008 12:21:44 +0000 Subject: test-suite/ideal-features/{apply.v -> eapply_evar.v} ...to avoid trouble on case-insensitive filesystems (Closes: #1987) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11531 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/ideal-features/apply.v | 9 --------- test-suite/ideal-features/eapply_evar.v | 9 +++++++++ 2 files changed, 9 insertions(+), 9 deletions(-) delete mode 100644 test-suite/ideal-features/apply.v create mode 100644 test-suite/ideal-features/eapply_evar.v (limited to 'test-suite/ideal-features') diff --git a/test-suite/ideal-features/apply.v b/test-suite/ideal-features/apply.v deleted file mode 100644 index b10d5dbf9..000000000 --- a/test-suite/ideal-features/apply.v +++ /dev/null @@ -1,9 +0,0 @@ -(* Test propagation of evars from subgoal to brother subgoals *) - -(* This does not work (oct 2008) because "match goal" sees "?evar = O" - and not "O = O" - -Lemma eapply_evar : O=O -> 0=O. -intro H; eapply trans_equal; - [apply H | match goal with |- ?x = ?x => reflexivity end]. -Qed. diff --git a/test-suite/ideal-features/eapply_evar.v b/test-suite/ideal-features/eapply_evar.v new file mode 100644 index 000000000..b10d5dbf9 --- /dev/null +++ b/test-suite/ideal-features/eapply_evar.v @@ -0,0 +1,9 @@ +(* Test propagation of evars from subgoal to brother subgoals *) + +(* This does not work (oct 2008) because "match goal" sees "?evar = O" + and not "O = O" + +Lemma eapply_evar : O=O -> 0=O. +intro H; eapply trans_equal; + [apply H | match goal with |- ?x = ?x => reflexivity end]. +Qed. -- cgit v1.2.3