diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-08-16 09:43:53 +0200 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-08-16 09:43:53 +0200 |
commit | 09b54382e52b572f8c091993309adcc4fea3a093 (patch) | |
tree | 941b56303eb6b9547702fe54e3650c27000d19f6 /test-suite | |
parent | 64061ae938b284f246586c2e7b959413953b4b0a (diff) | |
parent | 0b0411c56cac33ccd9474da4ae71d498355422b3 (diff) |
Merge PR #942: solving b1859
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/1859.v | 20 |
1 files changed, 20 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/1859.v b/test-suite/bugs/closed/1859.v new file mode 100644 index 000000000..43acfe4ba --- /dev/null +++ b/test-suite/bugs/closed/1859.v @@ -0,0 +1,20 @@ +Require Import Ring. +Require Import ArithRing. + +Ltac ring_simplify_neq := + match goal with + | [ H: ?X <> ?Y |- _ ] => progress ring_simplify X Y in H + end. + +Lemma toto : forall x y, x*1 <> y*1 -> y*1 <> x*1 -> x<>y. +Proof. + intros. + ring_simplify_neq. + ring_simplify_neq. + (* make sure ring_simplify has simplified both hypotheses *) + match goal with + | [ H: context[_*1] |- _ ] => fail 1 + | _ => idtac + end. + auto. +Qed. |