aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Specif.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-10 18:14:09 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 21:55:46 +0200
commit5bed8869b90510f719dcaa5e365b81c6309bdfff (patch)
tree2cfd060b65575d820598c8ce5a80cc18d875b7d0 /theories/Init/Specif.v
parentc4ce1baa9f66210ebc1909988b3dd8baa1b8ef27 (diff)
Adding option "Set Reversible Pattern Implicit" to Specif.v so that an
implicit is found whether one writes (sig P) or {x|P x}.
Diffstat (limited to 'theories/Init/Specif.v')
-rw-r--r--theories/Init/Specif.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index 6c0221856..d1038186e 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -9,6 +9,7 @@
(** Basic specifications : sets that may contain logical information *)
Set Implicit Arguments.
+Set Reversible Pattern Implicit.
Require Import Notations.
Require Import Datatypes.