aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-04-15 15:53:21 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-04-15 15:53:21 +0000
commit7ffd9e720a7e615bd5a55c9e1a6674d3b69ba177 (patch)
tree2d34d56c45840721436312890c7aa960b397ed46 /theories7
parentc8195deceaed2c8b98934b50870bf4a4dbc8139f (diff)
Bug réaffichage EXT
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5678 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Init/Logic_Type.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/theories7/Init/Logic_Type.v b/theories7/Init/Logic_Type.v
index 6fc763807..b57484801 100755
--- a/theories7/Init/Logic_Type.v
+++ b/theories7/Init/Logic_Type.v
@@ -72,8 +72,10 @@ Notation exT_intro := ex_intro (only parsing).
Notation exT_ind := ex_ind (only parsing).
Notation ExT := (ex ?).
-Notation "'EXT' x | p" := (ex ? [x]p) (at level 10, p at level 8).
-Notation "'EXT' x : t | p" := (ex ? [x:t]p) (at level 10, p at level 8).
+Notation "'EXT' x | p" := (ex ? [x]p)
+ (at level 10, p at level 8, only parsing).
+Notation "'EXT' x : t | p" := (ex ? [x:t]p)
+ (at level 10, p at level 8, only parsing).
(*
Inductive exT2 [A:Type;P,Q:A->Prop] : Prop
@@ -201,10 +203,10 @@ Notation identityT := identity (only parsing).
Notation refl_identityT := refl_identity (only parsing).
Notation "< A > x === y" := (!identityT A x y)
- (A annot, at level 1, x at level 0, only parsing).
+ (A annot, at level 1, x at level 0, only parsing) : type_scope.
Notation "x === y" := (identityT ? x y)
- (at level 5, no associativity) : type_scope.
+ (at level 5, no associativity, only parsing) : type_scope.
(*
Hints Resolve refl_identityT : core v62.