From 4ac0580306ea9e45da1863316936d700969465ad Mon Sep 17 00:00:00 2001 From: filliatr Date: Wed, 11 Apr 2001 12:41:41 +0000 Subject: documentation automatique de la bibliothèque standard MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1578 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Init/Peano.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Init/Peano.v') diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v index fc99d1a48..dcfbe5e99 100755 --- a/theories/Init/Peano.v +++ b/theories/Init/Peano.v @@ -131,7 +131,7 @@ Inductive le [n:nat] : nat -> Prop | le_S : (m:nat)(le n m)->(le n (S m)). Hint constr_le : core v62 := Constructors le. -(* equivalent to : "Hints Resolve le_n le_S : core v62." *) +(*i equivalent to : "Hints Resolve le_n le_S : core v62." i*) Definition lt := [n,m:nat](le (S n) m). Hints Unfold lt : core v62. -- cgit v1.2.3