src/HOL/Auth/Recur.ML
changeset 3516 470626799511
parent 3483 6988394a6008
child 3519 ab0a9fbed4c0
--- a/src/HOL/Auth/Recur.ML	Fri Jul 11 13:30:01 1997 +0200
+++ b/src/HOL/Auth/Recur.ML	Fri Jul 11 13:32:39 1997 +0200
@@ -74,15 +74,6 @@
 
 (**** Inductive proofs about recur ****)
 
-(*Monotonicity*)
-goal thy "!!evs. lost' <= lost ==> recur lost' <= recur lost";
-by (rtac subsetI 1);
-by (etac recur.induct 1);
-by (REPEAT_FIRST
-    (blast_tac (!claset addIs (impOfSubs(sees_mono RS analz_mono RS synth_mono)
-                              :: recur.intrs))));
-qed "recur_mono";
-
 (*Nobody sends themselves messages*)
 goal thy "!!evs. evs : recur lost ==> ALL A X. Says A A X ~: set evs";
 by (etac recur.induct 1);
@@ -490,21 +481,6 @@
 qed "Spy_not_see_session_key";
 
 
-goal thy 
- "!!evs. [| Crypt (shrK A) {|Key K, Agent A', N|}         \
-\              : parts(sees lost Spy evs);                \
-\           C ~: {A,A',Server};                           \
-\           A ~: lost;  A' ~: lost;  evs : recur lost |]  \
-\        ==> Key K ~: analz (sees lost C evs)";
-by (rtac (subset_insertI RS sees_mono RS analz_mono RS contra_subsetD) 1);
-by (rtac (sees_lost_agent_subset_sees_Spy RS analz_mono RS contra_subsetD) 1);
-by (FIRSTGOAL (rtac Spy_not_see_session_key));
-by (REPEAT_FIRST
-    (blast_tac
-     (!claset addIs (map impOfSubs [recur_mono, parts_mono, sees_mono]))));
-qed "Agent_not_see_session_key";
-
-
 (**** Authenticity properties for Agents ****)
 
 (*The response never contains Hashes*)