aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-05-15 20:13:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-05-15 20:13:06 +0000
commit76ed85857b467d38200a75b3dc7cd02d2d48b063 (patch)
treedb437c28061e8ccd24471e84cb280c7befacee43 /tactics
parent063831618cf9d7385fb6ba3f41dea102115f0fbc (diff)
Nouvelle syntaxe 'Match Reverse Context' pour garder un filtrage de
gauche à droite des hypothèses dans Intuition git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2696 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 7f29b4358..e193b20a9 100644
--- a/tactics/tauto.ml4
+++ b/tactics/tauto.ml4
@@ -55,7 +55,7 @@ let axioms ist =
let t_is_unit = tacticIn is_unit
and t_is_empty = tacticIn is_empty in
<:tactic<
- Match Context With
+ Match Reverse Context With
|[|- ?1] -> $t_is_unit;Constructor
|[_:?1 |- ?] -> $t_is_empty
|[_:?1 |- ?1] -> Assumption>>
@@ -68,7 +68,7 @@ let simplif t_reduce ist =
<:tactic<
$t_not_dep_intros;
Repeat
- ((Match Context With
+ ((Match Reverse Context With
| [id: (?1 ? ?) |- ?] ->
$t_is_conj;Elim id;Do 2 Intro;Clear id;$t_reduce
| [id: (?1 ? ?) |- ?] -> $t_is_disj;Elim id;Intro;Clear id;$t_reduce
@@ -94,7 +94,7 @@ let rec tauto_intuit t_reduce t_solver ist =
$t_reduce;
($t_simplif;$t_axioms
Orelse
- (Match Context With
+ (Match Reverse Context With
| [id:(?1-> ?2)-> ?3|- ?] ->
Cut ?2-> ?3;[Intro;Cut ?1-> ?2;[Intro;Cut ?3;[Intro;Clear id|
Intros;Apply id;Assumption]|Clear id]|Intros;Apply id;Try Intro;