diff -r ace45a11a45e -r bad75618fb82 src/HOL/Auth/Guard/P2.thy --- a/src/HOL/Auth/Guard/P2.thy Thu Jul 02 08:49:04 2020 +0000 +++ b/src/HOL/Auth/Guard/P2.thy Thu Jul 02 12:10:58 2020 +0000 @@ -193,6 +193,7 @@ lemma insertion_resilience: "\L. L \ valid A n B \ Suc i < len L \ ins (L,Suc i,M) \ valid A n B" +supply [[simproc del: defined_all]] apply (induct i) (* i = 0 *) apply clarify @@ -393,6 +394,7 @@ lemma pro_imp_Guard [rule_format]: "[| evs \ p2; B \ bad; A \ bad |] ==> pro B ofr A r I (cons M L) J C \ set evs \ Guard ofr {priK A} (spies evs)" +supply [[simproc del: defined_all]] apply (erule p2.induct) (* +3 subgoals *) (* Nil *) apply simp