diff src/MoreSpecif.v @ 142:6a00d49e85fb

Start of Reflection
author Adam Chlipala <adamc@hcoop.net>
date Tue, 28 Oct 2008 11:29:14 -0400
parents 939add5a7db9
children 5ea9a0bff8f7
line wrap: on
line diff
--- a/src/MoreSpecif.v	Mon Oct 27 10:31:57 2008 -0400
+++ b/src/MoreSpecif.v	Tue Oct 28 11:29:14 2008 -0400
@@ -73,3 +73,22 @@
 
 Notation "e1 ;;; e2" := (if e1 then e2 else !!)
   (right associativity, at level 60) : specif_scope.
+
+
+Section partial.
+  Variable P : Prop.
+
+  Inductive partial : Set :=
+  | Proved : P -> partial
+  | Uncertain : partial.
+End partial.
+
+Notation "[ P ]" := (partial P) : type_scope.
+
+Notation "'Yes'" := (Proved _) : partial_scope.
+Notation "'No'" := (Uncertain _) : partial_scope.
+
+Open Local Scope partial_scope.
+Delimit Scope partial_scope with partial.
+
+Notation "'Reduce' v" := (if v then Yes else No) : partial_scope.