aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes/SetoidDec.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-01-30 04:20:43 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-01-30 04:20:43 +0000
commit90b063be6b3c23a54e1d59974e09ee14f2941338 (patch)
tree65756ed843f1df72d9885d6450559aa120bc65b7 /theories/Classes/SetoidDec.v
parentbf4ea1d3edb56f9f63da38d08dd9fc14f5f9a4a3 (diff)
Support for occurences and 'in' in class_setoid, work on corresponding tactics in SetoidClass
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10486 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Classes/SetoidDec.v')
-rw-r--r--theories/Classes/SetoidDec.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/theories/Classes/SetoidDec.v b/theories/Classes/SetoidDec.v
index 3b4d90a5c..f68a7d3a4 100644
--- a/theories/Classes/SetoidDec.v
+++ b/theories/Classes/SetoidDec.v
@@ -22,6 +22,14 @@ Unset Strict Implicit.
Require Export Coq.Classes.SetoidClass.
+(** The [DecidableSetoid] class asserts decidability of a [Setoid]. It can be useful in proofs to reason more
+ classically. *)
+
+Require Import Coq.Logic.Decidable.
+
+Class [ Setoid A R ] => DecidableSetoid :=
+ setoid_decidable : forall x y : A, decidable (x == y).
+
(** The [EqDec] class gives a decision procedure for a particular setoid equality. *)
Class [ Setoid A R ] => EqDec :=