aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:04 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:04 +0200
commitee374eb0bbf32f192f474be25ad23bd21604d583 (patch)
tree7e32910be8528987dcb29e4606672cdebead9732 /theories/Init
parent155887217ff05af033840ded9c08ee40b19cac06 (diff)
Revert "Adding option "Set Reversible Pattern Implicit" to Specif.v so that an"
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/Specif.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index d1038186e..6c0221856 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -9,7 +9,6 @@
(** Basic specifications : sets that may contain logical information *)
Set Implicit Arguments.
-Set Reversible Pattern Implicit.
Require Import Notations.
Require Import Datatypes.