diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2011-03-05 16:42:21 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2011-03-05 16:42:21 +0000 |
commit | 4e5c9882c74b04e69ef885db7c05ed31bf6a2732 (patch) | |
tree | 4e6f41225aab90a0a6c70172e56b36e0cd07a058 /test-suite | |
parent | 627a69094f6126aeb1d959b6f610e865ebde8a73 (diff) |
Improved define_evar_as_lambda which was creating an unrelated new evar
for the domain instead of retrieving the known domain of the initial evar.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13881 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/success/evars.v | 4 |
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/success/evars.v b/test-suite/success/evars.v index 69f7164c7..52c4f2daa 100644 --- a/test-suite/success/evars.v +++ b/test-suite/success/evars.v @@ -254,3 +254,7 @@ Proof. (* error message with V8.3 : Impossible to unify "?18" with "fun g : nat -> nat => ?6 = g". *) Abort. + +(* Regression test *) + +Definition fo : option nat -> nat := option_rec _ (fun a => 0) 0. |