src/HOL/UNITY/Guar.ML
changeset 7878 43b03d412b82
parent 7689 affe0c2fdfbf
child 7947 b999c1ab9327
--- a/src/HOL/UNITY/Guar.ML	Mon Oct 18 15:17:35 1999 +0200
+++ b/src/HOL/UNITY/Guar.ML	Mon Oct 18 15:18:24 1999 +0200
@@ -65,7 +65,7 @@
 (*** guarantees ***)
 
 val prems = Goal
-     "(!!G. [| F Join G : X;  Disjoint F G |] ==> F Join G : Y) \
+     "(!!G. [| F Join G : X;  Disjoint UNIV F G |] ==> F Join G : Y) \
 \     ==> F : X guarantees Y";
 by (simp_tac (simpset() addsimps [guar_def, component_eq]) 1);
 by (blast_tac (claset() addIs prems) 1);
@@ -84,7 +84,7 @@
 
 (*This equation is more intuitive than the official definition*)
 Goal "(F : X guarantees Y) = \
-\     (ALL G. F Join G : X & Disjoint F G --> F Join G : Y)";
+\     (ALL G. F Join G : X & Disjoint UNIV F G --> F Join G : Y)";
 by (simp_tac (simpset() addsimps [guar_def, component_eq]) 1);
 by (Blast_tac 1);
 qed "guarantees_eq";