# HG changeset patch # User paulson # Date 988883622 -7200 # Node ID f2a284b2d5887d18a7ab6b9322831d6b96f94858 # Parent 6fdc4c4ccec185ae1d6fbba4045c54ff517bf2b1 minor tweaks diff -r 6fdc4c4ccec1 -r f2a284b2d588 src/HOL/Auth/Recur.thy --- a/src/HOL/Auth/Recur.thy Thu May 03 10:27:37 2001 +0200 +++ b/src/HOL/Auth/Recur.thy Thu May 03 11:53:42 2001 +0200 @@ -131,7 +131,7 @@ lemma "\K. \NA. \evs \ recur. Says B A {|Crypt (shrK A) {|Key K, Agent B, Nonce NA|}, END|} \ set evs" -apply (tactic "cut_facts_tac [Nonce_supply2, Key_supply2] 1") +apply (cut_tac Nonce_supply2 Key_supply2) apply clarify apply (intro exI bexI) apply (rule_tac [2] @@ -253,7 +253,7 @@ (K \ KK | Key K \ analz (spies evs))" apply (erule recur.induct) apply (drule_tac [4] RA2_analz_spies, - frule_tac [5] respond_imp_responses, + drule_tac [5] respond_imp_responses, drule_tac [6] RA4_analz_spies) apply analz_freshK apply spy_analz @@ -285,9 +285,9 @@ evs \ recur; A \ bad |] ==> X \ parts (spies evs)" apply (erule rev_mp) apply (erule recur.induct, - frule_tac [6] RA4_parts_spies, - frule_tac [5] respond_imp_responses, - frule_tac [4] RA2_parts_spies) + drule_tac [6] RA4_parts_spies, + drule_tac [5] respond_imp_responses, + drule_tac [4] RA2_parts_spies) (*RA3 requires a further induction*) apply (erule_tac [5] responses.induct) apply simp_all @@ -311,7 +311,7 @@ ==> B=B' & P=P'" apply (erule rev_mp, erule rev_mp) apply (erule recur.induct, - frule_tac [5] respond_imp_responses) + drule_tac [5] respond_imp_responses) apply (force, simp_all) (*Fake*) apply blast @@ -464,13 +464,13 @@ apply (unfold HPair_def) apply (erule rev_mp) apply (erule recur.induct, - frule_tac [6] RA4_parts_spies, - frule_tac [4] RA2_parts_spies, + drule_tac [6] RA4_parts_spies, + drule_tac [4] RA2_parts_spies, simp_all) (*Nil*) apply force (*Fake, RA3*) -apply (blast dest: Hash_in_parts_respond)+; +apply (blast dest: Hash_in_parts_respond)+ done (** These two results subsume (for all agents) the guarantees proved