src/ZF/UNITY/Follows.ML
changeset 14053 4daa384f4fd7
parent 14052 e9c9f69e4f63
child 14055 a3f592e3f4bd
--- a/src/ZF/UNITY/Follows.ML	Wed May 28 18:13:41 2003 +0200
+++ b/src/ZF/UNITY/Follows.ML	Thu May 29 17:10:00 2003 +0200
@@ -8,6 +8,10 @@
  
 (*Does this hold for "invariant"?*)
 
+val prems =
+Goal "[|A=A'; r=r'; !!x. x:state ==> f(x)=f'(x); !!x. x:state ==> g(x)=g'(x)|] ==> Follows(A, r, f, g) = Follows(A', r', f', g')";
+by (asm_full_simp_tac (simpset() addsimps [Increasing_def,Follows_def]@prems) 1);
+qed "Follows_cong";
 
 Goalw [mono1_def, comp_def] 
 "[| mono1(A, r, B, s, h); ALL x:state. f(x):A & g(x):A |] ==> \