diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/SET_Protocol/Message_SET.thy --- a/src/HOL/SET_Protocol/Message_SET.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/SET_Protocol/Message_SET.thy Sat Jan 05 17:24:33 2019 +0100 @@ -21,12 +21,12 @@ text\Collapses redundant cases in the huge protocol proofs\ lemmas disj_simps = disj_comms disj_left_absorb disj_assoc -text\Effective with assumptions like @{term "K \ range pubK"} and - @{term "K \ invKey`range pubK"}\ +text\Effective with assumptions like \<^term>\K \ range pubK\ and + \<^term>\K \ invKey`range pubK\\ lemma notin_image_iff: "(y \ f`I) = (\i\I. f i \ y)" by blast -text\Effective with the assumption @{term "KK \ - (range(invKey o pubK))"}\ +text\Effective with the assumption \<^term>\KK \ - (range(invKey o pubK))\\ lemma disjoint_image_iff: "(A \ - (f`I)) = (\i\I. f i \ A)" by blast @@ -263,7 +263,7 @@ text\This allows \blast\ to simplify occurrences of - @{term "parts(G\H)"} in the assumption.\ + \<^term>\parts(G\H)\ in the assumption.\ declare parts_Un [THEN equalityD1, THEN subsetD, THEN UnE, elim!]