aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Setoids
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-04-17 11:30:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-04-17 11:30:23 +0000
commitcc1be0bf512b421336e81099aa6906ca47e4257a (patch)
treec25fa8ed965729d7a85efa3b3292fdf7f442963d /theories/Setoids
parentebf9aa9f97ef0d49ed1b799c9213f78efad4fec7 (diff)
Uniformisation (Qed/Save et Implicits Arguments)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2650 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Setoids')
-rw-r--r--theories/Setoids/Setoid.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/Setoids/Setoid.v b/theories/Setoids/Setoid.v
index 4e33e4728..0807f93b9 100644
--- a/theories/Setoids/Setoid.v
+++ b/theories/Setoids/Setoid.v
@@ -25,7 +25,7 @@ End Setoid.
Definition Prop_S : (Setoid_Theory Prop iff).
Split; [Exact iff_refl | Exact iff_sym | Exact iff_trans].
-Save.
+Qed.
Add Setoid Prop iff Prop_S.
@@ -43,7 +43,7 @@ Apply (H3 H2).
Right.
Inversion H0.
Apply (H3 H2).
-Save.
+Qed.
Add Morphism and : and_ext.
Intros.
@@ -54,14 +54,14 @@ Apply (H4 H2).
Inversion H0.
Apply (H4 H3).
-Save.
+Qed.
Add Morphism not : not_ext.
Red ; Intros.
Apply H0.
Inversion H.
Apply (H3 H1).
-Save.
+Qed.
Definition fleche [A,B:Prop] := A -> B.
@@ -71,5 +71,5 @@ Intros.
Inversion H0.
Inversion H.
Apply (H3 (H1 (H6 H2))).
-Save.
+Qed.