aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/unification.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-15 12:00:50 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-15 12:00:50 +0000
commit07e03e167c7eda30ffc989530470b5c597beaedc (patch)
tree5bee610e35b3110430622cd1573d4971f70d28e4 /test-suite/success/unification.v
parenta036149469ef4c37e77018b1d47d24edfced6e04 (diff)
- Un peu de doc, préparation du CHANGES pour la release.
- Re-restriction de inversion (après la correction des bugs - et notamment du "Unknown meta" qui apparaissait parfois -, inversion devenait capable d'agir sur des buts non atomiques, ce qui crée quelques incompatibilités, typiquement dans CoRN où inversion est utilisé dans un rôle de discriminate; en attendant de voir, on revient à la sémantique initiale). - Généralisation de Local/Global dans Implicit Arguments pour avoir un fonctionnement plus uniforme et plus facile à documenter. - Code mort (clenv.ml). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10796 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/unification.v')
-rw-r--r--test-suite/success/unification.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index e31d67d8c..51b0e06e5 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -109,3 +109,11 @@ intros.
apply H0. (* Check that equation ?n[H] = ?n[H] is correctly considered true *)
reflexivity.
Qed.
+
+(* Check treatment of metas erased by K-redexes at the time of turning
+ them to evas *)
+
+Inductive nonemptyT (t : Type) : Prop := nonemptyT_intro : t -> nonemptyT t.
+Goal True.
+try case nonemptyT_intro. (* check that it fails w/o anomaly *)
+Abort.