src/HOL/UNITY/Constrains.thy
changeset 5784 54276fba8420
parent 5648 fe887910e32e
child 6535 880f31a62784
equal deleted inserted replaced
5783:95ac0bf10518 5784:54276fba8420
    21     "Unless A B == Constrains (A-B) (A Un B)"
    21     "Unless A B == Constrains (A-B) (A Un B)"
    22 
    22 
    23   Invariant :: "'a set => 'a program set"
    23   Invariant :: "'a set => 'a program set"
    24     "Invariant A == {F. Init F <= A} Int Stable A"
    24     "Invariant A == {F. Init F <= A} Int Stable A"
    25 
    25 
       
    26   (*Polymorphic in both states and the meaning of <= *)
       
    27   Increasing :: "['a => 'b::{ord}] => 'a program set"
       
    28     "Increasing f == INT z. Stable {s. z <= f s}"
       
    29 
    26 end
    30 end