From ec3bff58d151ff804866175e907664d1fba3c600 Mon Sep 17 00:00:00 2001 From: pboutill Date: Thu, 9 Aug 2012 21:57:29 +0000 Subject: Unification in Evar_conv uses an abstract machine state It uses a term in front of a stack instead of a term in front of a list of applied terms. From outside of eq_appr_x nothing should have changed. Nasty evar instantiation bug git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15719 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/success/unification.v | 4 ++++ 1 file changed, 4 insertions(+) (limited to 'test-suite') diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v index 997dceb4d..249079294 100644 --- a/test-suite/success/unification.v +++ b/test-suite/success/unification.v @@ -1,3 +1,7 @@ +Let test_stack_unification_interaction_with_delta A + : (if negb _ then true else false) = if orb false (negb A) then true else false + := eq_refl. + (* Test patterns unification *) Lemma l1 : (forall P, (exists x:nat, P x) -> False) -- cgit v1.2.3