aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-20 18:10:57 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-20 18:10:57 +0000
commit1f96d480842a1206a9334d0c8b1b6cc4647066ef (patch)
tree9fc22a20d49bcefca1d863aee9d36c5fab03334f /theories
parent6c7f6fa6c215e5e28fcf23bf28ccb9db543709ba (diff)
Transparent
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2035 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rwxr-xr-xtheories/Arith/Peano_dec.v6
-rwxr-xr-xtheories/Init/Logic.v9
2 files changed, 9 insertions, 6 deletions
diff --git a/theories/Arith/Peano_dec.v b/theories/Arith/Peano_dec.v
index d847a060d..694351b67 100755
--- a/theories/Arith/Peano_dec.v
+++ b/theories/Arith/Peano_dec.v
@@ -15,17 +15,17 @@ Proof.
NewInduction n.
Auto.
Left; Exists n; Auto.
-Qed.
+Defined.
Theorem eq_nat_dec : (n,m:nat){n=m}+{~(n=m)}.
Proof.
NewInduction n; NewInduction m; Auto.
Elim (IHn m); Auto.
-Qed.
+Defined.
Hints Resolve O_or_S eq_nat_dec : arith.
Theorem dec_eq_nat:(x,y:nat)(decidable (x=y)).
Intros x y; Unfold decidable; Elim (eq_nat_dec x y); Auto with arith.
-Qed.
+Defined.
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 14f331930..645f4b0d7 100755
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -139,17 +139,20 @@ Section Logic_lemmas.
Theorem sym_eq : (eq ? x y) -> (eq ? y x).
Proof.
Induction 1; Trivial.
- Qed.
+ Defined.
+ Opaque sym_eq.
Theorem trans_eq : (eq ? x y) -> (eq ? y z) -> (eq ? x z).
Proof.
Induction 2; Trivial.
- Qed.
+ Defined.
+ Opaque trans_eq.
Theorem f_equal : (eq ? x y) -> (eq ? (f x) (f y)).
Proof.
Induction 1; Trivial.
- Qed.
+ Defined.
+ Opaque f_equal.
Theorem sym_not_eq : (not (eq ? x y)) -> (not (eq ? y x)).
Proof.