diff options
| author | delahaye | 2001-06-15 21:54:45 +0000 |
|---|---|---|
| committer | delahaye | 2001-06-15 21:54:45 +0000 |
| commit | 686b7d347ba8dc9a4e032cd4c6cb38da93c38188 (patch) | |
| tree | 9a460732642bee4e80140d0db3d1e825015ee929 | |
| parent | 560dd7089c3f5304db9596486ea423484f86c891 (diff) | |
Fix d'un bug de Tauto
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1787 85f007b7-540e-0410-9357-904b9bb8a0f7
| -rw-r--r-- | tactics/tauto.ml4 | 6 | ||||
| -rw-r--r-- | test-suite/success/Tauto.v | 7 |
2 files changed, 10 insertions, 3 deletions
diff --git a/tactics/tauto.ml4 b/tactics/tauto.ml4 index ffb7f09a15..1788298be9 100644 --- a/tactics/tauto.ml4 +++ b/tactics/tauto.ml4 @@ -79,8 +79,8 @@ let simplif () = $t_is_conj;Cut ?2-> ?3-> ?4;[Intro;Clear id|Intros;Apply id; Try Split;Assumption] | [id: (?1 ?2 ?3) -> ?4|- ?] -> - $t_is_disj;Cut ?3-> ?4;[Cut ?2-> ?4;[Intros;Clear id|Intro;Apply id; - Left;Assumption]|Intro;Apply id;Right;Assumption] + $t_is_disj;Cut ?3-> ?4;[Cut ?2-> ?4;[Intros;Clear id|Intros;Apply id; + Try Left;Assumption]|Intros;Apply id;Try Right;Assumption] | [id0: ?1-> ?2; id1: ?1|- ?] -> Generalize (id0 id1);Intro;Clear id0 | [id: ?1 -> ?2|- ?] -> $t_is_unit;Cut ?2;[Intro;Clear id|Intros;Apply (id I);Assumption] @@ -97,7 +97,7 @@ let rec tauto_main () = (Match 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;Intro; + Intros;Apply id;Assumption]|Clear id]|Intros;Apply id;Try Intro; Assumption];$t_tauto_main | [|- (?1 ? ?)] -> $t_is_disj;(Left;$t_tauto_main) Orelse (Right;$t_tauto_main)) diff --git a/test-suite/success/Tauto.v b/test-suite/success/Tauto.v index 6e8bf0f140..ecaaf80d4f 100644 --- a/test-suite/success/Tauto.v +++ b/test-suite/success/Tauto.v @@ -172,6 +172,13 @@ Proof. Tauto. Save. +(* A bug from CNF form *) +Lemma old_bug3: + ((~A\/B)/\(~B\/B)/\(~A\/~B)/\(~B\/~B)->False)->~((A->B)->B)->False. +Proof. + Tauto. +Save. + (* A private club has the following rules : * * . rule 1 : Every non-scottish member wears red socks |
