diff options
author | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2017-04-10 16:37:11 +0200 |
---|---|---|
committer | Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr> | 2017-04-10 16:40:20 +0200 |
commit | d331543b7b759bb97ea1ece32501cd0149627e9f (patch) | |
tree | 700e524eaaa5a4a4519454024046fe379e516df3 /test-suite/success | |
parent | 1d3500af261d01ec552424c46311d49fe61c1300 (diff) |
Adding a test for the correctness of normalization in legacy typeclasses.
This is a test for commit 9d1230d484a2cf519f9cd76dc0f37815f3c6339b.
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/old_typeclass.v | 13 |
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/success/old_typeclass.v b/test-suite/success/old_typeclass.v new file mode 100644 index 000000000..01e35810b --- /dev/null +++ b/test-suite/success/old_typeclass.v @@ -0,0 +1,13 @@ +Require Import Setoid Coq.Classes.Morphisms. +Set Typeclasses Legacy Resolution. + +Declare Instance and_Proper_eq: Proper (Logic.eq ==> Logic.eq ==> Logic.eq) and. + +Axiom In : Prop. +Axiom union_spec : In <-> True. + +Lemma foo : In /\ True. +Proof. +progress rewrite union_spec. +repeat constructor. +Qed. |