From b91f721df622b40e1f4ca610dd4a5697d27ec56a Mon Sep 17 00:00:00 2001 From: herbelin Date: Tue, 25 Oct 2011 21:02:50 +0000 Subject: Merge common notations from Utf8.v and Utf8_core.v (see bug report #2610). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14605 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Unicode/Utf8.v | 17 +---------------- theories/Unicode/Utf8_core.v | 2 ++ 2 files changed, 3 insertions(+), 16 deletions(-) (limited to 'theories/Unicode') diff --git a/theories/Unicode/Utf8.v b/theories/Unicode/Utf8.v index 7f35088bc..4d44dd85c 100644 --- a/theories/Unicode/Utf8.v +++ b/theories/Unicode/Utf8.v @@ -7,22 +7,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* Logic *) -Notation "∀ x .. y , P" := (forall x, .. (forall y, P) ..) - (at level 200, x binder, y binder, right associativity) : type_scope. -Notation "∃ x .. y , P" := (exists x, .. (exists y, P) ..) - (at level 200, x binder, y binder, right associativity) : type_scope. - -Notation "x ∨ y" := (x \/ y) (at level 85, right associativity) : type_scope. -Notation "x ∧ y" := (x /\ y) (at level 80, right associativity) : type_scope. -Notation "x → y" := (x -> y) (at level 90, right associativity): type_scope. -Notation "x ↔ y" := (x <-> y) (at level 95, no associativity): type_scope. -Notation "¬ x" := (~x) (at level 75, right associativity) : type_scope. -Notation "x ≠ y" := (x <> y) (at level 70) : type_scope. - -(* Abstraction *) -Notation "'λ' x .. y , t" := (fun x => .. (fun y => t) ..) - (at level 200, x binder, y binder, right associativity). +Require Import Utf8_core. (* Arithmetic *) Notation "x ≤ y" := (le x y) (at level 70, no associativity). diff --git a/theories/Unicode/Utf8_core.v b/theories/Unicode/Utf8_core.v index a42de3abd..31724b3ca 100644 --- a/theories/Unicode/Utf8_core.v +++ b/theories/Unicode/Utf8_core.v @@ -7,6 +7,8 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) + + (* Logic *) Notation "∀ x .. y , P" := (forall x, .. (forall y, P) ..) (at level 200, x binder, y binder, right associativity) : type_scope. -- cgit v1.2.3