aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2018-02-23 15:34:26 +0100
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2018-03-04 19:40:22 +0100
commit84e9fc5da618e9e2248ba4a650b07b6b5528f957 (patch)
treefef97f79ef48048c98e6ca2c5238d544e3294dc7 /test-suite/success
parent78551857a41a57607ecfb3fd010e0a9755f47cea (diff)
Remove deprecated options related to typeclasses.
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/old_typeclass.v13
1 files changed, 0 insertions, 13 deletions
diff --git a/test-suite/success/old_typeclass.v b/test-suite/success/old_typeclass.v
deleted file mode 100644
index 01e35810b..000000000
--- a/test-suite/success/old_typeclass.v
+++ /dev/null
@@ -1,13 +0,0 @@
-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.