From 7e52301b501f7a574fca19776fb7fcbfe873d533 Mon Sep 17 00:00:00 2001 From: herbelin Date: Tue, 30 Mar 2010 21:26:06 +0000 Subject: Small things about coqdoc + fixing lettuple.v test (part of bug #2289) In coqdoc, made links to utf8 notations working and made representation of locations for notations more compact git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12896 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/coqdoc/links.v | 8 +++++--- 1 file changed, 5 insertions(+), 3 deletions(-) (limited to 'test-suite/coqdoc') diff --git a/test-suite/coqdoc/links.v b/test-suite/coqdoc/links.v index b09d64a9a..16028fe17 100644 --- a/test-suite/coqdoc/links.v +++ b/test-suite/coqdoc/links.v @@ -19,7 +19,9 @@ Notation "n ++ m" := (plus n m). Notation "n ++ m" := (mult n m). (* redefinition *) -Notation "n % m" := (plus n m) (at level 60). +Notation "n ** m" := (plus n m) (at level 60). + +Notation "n ▵ m" := (plus n m) (at level 60). Notation "n '_' ++ 'x' m" := (plus n m) (at level 3). @@ -31,7 +33,7 @@ Definition eq0 := 0 = 0 :> nat. Notation "( x # y ; .. ; z )" := (pair .. (pair x y) .. z). -Definition p := ((0#0;0) , (0 % 0)). +Definition b_α := ((0#0;0) , (0 ** 0)). Notation h := a. @@ -39,7 +41,7 @@ Notation h := a. Variables b' b2: nat. - Notation "n + m" := (plus n m) : my_scope. + Notation "n + m" := (n ▵ m) : my_scope. Delimit Scope my_scope with my. -- cgit v1.2.3