aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-08-26 13:11:25 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-08-26 13:11:25 +0000
commitf43d75830bec7ce179ca11a8eb1baf9381383bf4 (patch)
tree1e0d701df691060240019dd1cc3465acd232fb45 /theories
parent349203bb70ac058df209137320548f918f15db25 (diff)
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7322 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Init/Tactics.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Tactics.v b/theories/Init/Tactics.v
index 89a319f09..f221aa8b4 100644
--- a/theories/Init/Tactics.v
+++ b/theories/Init/Tactics.v
@@ -45,7 +45,7 @@ Ltac f_equal :=
let des := destruct 1 || intro in
let r := try reflexivity in
match goal with
- | |- ?f ?a = ?f' ?a' => cut (a=a'); des; r
+ | |- ?f ?a = ?f' ?a' => cut (a=a'); [des; r|r]
| |- ?f ?a ?b = ?f' ?a' ?b' =>
cut (b=b');[cut (a=a');[do 2 des; r|r]|r]
| |- ?f ?a ?b ?c = ?f' ?a' ?b' ?c'=>