src/HOL/UNITY/Constrains.ML
changeset 8216 e4b3192dfefa
parent 8069 19b9f92ca503
child 8334 7896bcbd8641
--- a/src/HOL/UNITY/Constrains.ML	Wed Feb 09 11:43:53 2000 +0100
+++ b/src/HOL/UNITY/Constrains.ML	Wed Feb 09 11:45:10 2000 +0100
@@ -203,6 +203,11 @@
 
 (*** Increasing ***)
 
+Goalw [Increasing_def]
+     "F : Increasing f ==> F : Stable {s. x <= f s}";
+by (Blast_tac 1);
+qed "IncreasingD";
+
 Goalw [Increasing_def, Stable_def, Constrains_def, stable_def, constrains_def]
      "mono g ==> Increasing f <= Increasing (g o f)";
 by Auto_tac;
@@ -210,10 +215,10 @@
 qed "mono_Increasing_o";
 
 Goalw [Increasing_def]
-     "Increasing f <= {F. ALL z::nat. F: Stable {s. z < f s}}";
+     "!!z::nat. F : Increasing f ==> F: Stable {s. z < f s}";
 by (simp_tac (simpset() addsimps [Suc_le_eq RS sym]) 1);
 by (Blast_tac 1);
-qed "Increasing_Stable_less";
+qed "strict_IncreasingD";
 
 Goalw [increasing_def, Increasing_def]
      "F : increasing f ==> F : Increasing f";