aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
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-06-16 17:30:18 +0200
commit3f768f404a36ebd3e2a5b10a9fe48e5122e4cd62 (patch)
tree0698756a2deee627225e8425ada7f85450bb612c /theories/Init
parente09062253640add21f395f688f927a26cf38106e (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')
-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.