aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-25 12:12:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-25 12:12:06 +0000
commitd0ee77343eeecae0ad314ea877c60b4dfa77ad41 (patch)
treef4a79dafb926d561f4334c5b0d757e12f7d74750
parent2fb6de71c225ebd8ebada632b3f45ee9c878ddc9 (diff)
Retablissement SynDef Value/Error
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3278 85f007b7-540e-0410-9357-904b9bb8a0f7
-rwxr-xr-xtheories/Init/Specif.v3
-rw-r--r--theories/Init/SpecifSyntax.v2
2 files changed, 3 insertions, 2 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index daf7e5d85..46203fe1f 100755
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -147,6 +147,9 @@ Definition Exc := option.
Definition value := Some.
Definition error := None.
+Syntactic Definition Error := (error ?).
+Syntactic Definition Value := (value ?).
+
Definition except := False_rec. (* for compatibility with previous versions *)
Theorem absurd_set : (A:Prop)(C:Set)A->(~A)->C.
diff --git a/theories/Init/SpecifSyntax.v b/theories/Init/SpecifSyntax.v
index a617373c8..af41b7208 100644
--- a/theories/Init/SpecifSyntax.v
+++ b/theories/Init/SpecifSyntax.v
@@ -22,8 +22,6 @@ Notation "A + { B }" := (sumor A B)
Notation ProjS1 := (projS1 ?).
Notation ProjS2 := (projS2 ?).
-Notation Error := (error ?).
-Notation Value := (value ?).
Notation Except := (except ?).
Notation "{ x : A | P }" := (sig A [x:A]P)