aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Setoids
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Setoids')
-rw-r--r--theories/Setoids/Setoid.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/theories/Setoids/Setoid.v b/theories/Setoids/Setoid.v
index 7d8196a72..1bf729055 100644
--- a/theories/Setoids/Setoid.v
+++ b/theories/Setoids/Setoid.v
@@ -608,9 +608,13 @@ Add Morphism not : Not_Morphism.
tauto.
Qed.
+Theorem impl_refl: reflexive _ impl.
+ hnf; unfold impl; tauto.
+Qed.
+
(* THE ASYMMETRIC AREFLEXIVE RELATION impl WITH A FEW MORPHISMS *)
-Add Relation Prop impl.
+Add Relation Prop impl reflexivity proved by impl_refl.
Add Morphism impl with signature impl --> impl ++> impl as Impl_Morphism2.
unfold impl; tauto.