aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-01-29 17:05:59 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-01-29 17:05:59 +0000
commit65fe36d2ad32f2c46c67369555aa5f3461570b78 (patch)
tree75673616a4ad43394696cda74c2a6f67b564c86a /tactics
parent627ab72099948f785920b5bc863cc9f5e9d9ad11 (diff)
Solves some warning and hides some not-bad ones in doc. It remains a
few hevea warning (failure to put a vector on an expression in Classes.tex, failure to support multirow in RecTutorial.tex). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11868 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tauto.ml46
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/tauto.ml4 b/tactics/tauto.ml4
index f7713f015..3f5b0a4a3 100644
--- a/tactics/tauto.ml4
+++ b/tactics/tauto.ml4
@@ -181,7 +181,7 @@ let simplif ist =
| id: ?X1 |- _ => $t_is_conj; elim id; do 2 intro; clear id
| id: (Coq.Init.Logic.iff _ _) |- _ => elim id; do 2 intro; clear id
| id: ?X1 |- _ => $t_is_disj; elim id; intro; clear id
- | id0: ?X1-> ?X2, id1: ?X1|- _ =>
+ | id0: ?X1 -> ?X2, id1: ?X1|- _ =>
(* generalize (id0 id1); intro; clear id0 does not work
(see Marco Maggiesi's bug PR#301)
so we instead use Assert and exact. *)
@@ -201,7 +201,7 @@ let simplif ist =
clear id
| id: ?X1 -> ?X2|- _ =>
$t_flatten_contravariant_disj
- (* moved from "id:(?A\/?B)->?X2|-" to "?A->?X2|-" and "?B->?X2|-" *)
+ (* moved from "id:(?A\/?B)->?X2|-" to "?A->?X2,?B->?X2|-" *)
| |- ?X1 => $t_is_conj; split
| |- (Coq.Init.Logic.iff _ _) => split
end;
@@ -216,7 +216,7 @@ let rec tauto_intuit t_reduce solver ist =
<:tactic<
($t_simplif;$t_axioms
|| match reverse goal with
- | id:(?X1-> ?X2)-> ?X3|- _ =>
+ | id:(?X1 -> ?X2)-> ?X3|- _ =>
cut X3;
[ intro; clear id; $t_tauto_intuit
| cut (X1 -> X2);