aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-21 12:47:51 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-21 12:47:51 +0000
commit41c74d93574d796535e5f89d52b9a53fd3017966 (patch)
treeea60058b7b498d780fc1ddc9c49baa36e0e23a84 /theories
parentd5fc85b0b69b870b9dde5cc3b8faa5cbb5251881 (diff)
separation calcul des implicites et declaration des constantes / inductifs / variables
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@897 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rwxr-xr-xtheories/Init/Logic.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 545c0acb7..ec1d850e0 100755
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -114,7 +114,7 @@ Section Logic_lemmas.
Variable x,y,z : A.
Theorem sym_eq : (eq ? x y) -> (eq ? y x).
- Proof.
+ Proof.
Induction 1; Trivial.
Qed.