aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Specif.v
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-07-26 11:30:17 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-07-26 11:30:17 +0000
commit433e283c473d7025bbb594fd871de1e7ab285e6b (patch)
treee94fa6a36f79cdfacc25f7f926444bc85f732571 /theories/Init/Specif.v
parent5c556a472e8d91a46760ad5dcf6dafb20846d7e7 (diff)
Same Implicit Arguments rule for sumbool and sumor.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14295 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Specif.v')
-rw-r--r--theories/Init/Specif.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index 602507867..12ac08ff0 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -139,6 +139,9 @@ Inductive sumor (A:Type) (B:Prop) : Type :=
Add Printing If sumor.
+Implicit Arguments inleft [[A] [B]] [A].
+Implicit Arguments inright [[A] [B]] [B].
+
(** Various forms of the axiom of choice for specifications *)
Section Choice_lemmas.