src/HOL/UNITY/UNITY.ML
changeset 6712 d1bebb7f1c50
parent 6536 281d44905cab
child 7240 a509730e424b
equal deleted inserted replaced
6711:d45359e7dcbf 6712:d1bebb7f1c50
   264 
   264 
   265 
   265 
   266 (*** increasing ***)
   266 (*** increasing ***)
   267 
   267 
   268 Goalw [increasing_def, stable_def, constrains_def]
   268 Goalw [increasing_def, stable_def, constrains_def]
   269      "increasing f <= increasing (length o f)";
   269      "mono g ==> increasing f <= increasing (g o f)";
   270 by Auto_tac;
   270 by Auto_tac;
   271 by (blast_tac (claset() addIs [prefix_length_le, le_trans]) 1);
   271 by (blast_tac (claset() addIs [monoD, order_trans]) 1);
   272 qed "increasing_size";
   272 qed "mono_increasing_o";
   273 
   273 
   274 Goalw [increasing_def]
   274 Goalw [increasing_def]
   275      "increasing f <= {F. ALL z::nat. F: stable {s. z < f s}}";
   275      "increasing f <= {F. ALL z::nat. F: stable {s. z < f s}}";
   276 by (simp_tac (simpset() addsimps [Suc_le_eq RS sym]) 1);
   276 by (simp_tac (simpset() addsimps [Suc_le_eq RS sym]) 1);
   277 by (Blast_tac 1);
   277 by (Blast_tac 1);