src/HOL/UNITY/Guar.ML
changeset 7947 b999c1ab9327
parent 7878 43b03d412b82
child 8055 bb15396278fb
--- a/src/HOL/UNITY/Guar.ML	Wed Oct 27 13:02:23 1999 +0200
+++ b/src/HOL/UNITY/Guar.ML	Wed Oct 27 13:03:32 1999 +0200
@@ -191,11 +191,6 @@
 by (Blast_tac 1);
 qed "guarantees_Join_Un";
 
-Goal "((JOIN I F) <= H) = (ALL i: I. F i <= H)";
-by (simp_tac (simpset() addsimps [component_eq_subset]) 1);
-by (Blast_tac 1);
-qed "JN_component_iff";
-
 Goalw [guar_def]
     "[| ALL i:I. F i : X i guarantees Y i |] \
 \    ==> (JOIN I F) : (INTER I X) guarantees (INTER I Y)";