aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Compat
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-04-05 12:56:52 -0400
committerGravatar Jason Gross <jgross@mit.edu>2016-04-05 13:01:59 -0400
commita585d46fbacfcc9cddf3da439e5f7001d429ba2a (patch)
tree67a7832dd74816fb400451a9bb19af1ccb9b28a5 /theories/Compat
parent4c078b0362542908eb2fe1d63f0d867b339953fd (diff)
Fix bug #4656
I introduced this bug in 4c078b0362542908eb2fe1d63f0d867b339953fd; Coq.Init.Notations.constructor does not take any arguments.
Diffstat (limited to 'theories/Compat')
-rw-r--r--theories/Compat/Coq84.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Compat/Coq84.v b/theories/Compat/Coq84.v
index 5036b9bc8..326628192 100644
--- a/theories/Compat/Coq84.v
+++ b/theories/Compat/Coq84.v
@@ -22,10 +22,11 @@ Global Set Nonrecursive Elimination Schemes.
Global Set Universal Lemma Under Conjunction.
(** In 8.4, [constructor (tac)] allowed backtracking across the use of [constructor]; it has been subsumed by [constructor; tac]. *)
+Ltac constructor_84_n n := constructor n.
Ltac constructor_84_tac tac := once (constructor; tac).
Tactic Notation "constructor" := Coq.Init.Notations.constructor.
-Tactic Notation "constructor" int_or_var(n) := Coq.Init.Notations.constructor n.
+Tactic Notation "constructor" int_or_var(n) := constructor_84_n n.
Tactic Notation "constructor" "(" tactic(tac) ")" := constructor_84_tac tac.
(** Some tactic notations do not factor well with tactics; we add global parsing entries for some tactics that would otherwise be overwritten by custom variants. See https://coq.inria.fr/bugs/show_bug.cgi?id=4392. *)
@@ -43,7 +44,6 @@ Tactic Notation "left" := left.
Tactic Notation "eleft" := eleft.
Tactic Notation "right" := right.
Tactic Notation "eright" := eright.
-Tactic Notation "constructor" := constructor.
Tactic Notation "econstructor" := econstructor.
Tactic Notation "symmetry" := symmetry.
Tactic Notation "split" := split.