src/HOL/UNITY/UNITY.thy
changeset 8948 b797cfa3548d
parent 6823 97babc436a41
child 10064 1a77667b21ef
equal deleted inserted replaced
8947:971aedd340e4 8948:b797cfa3548d
     6 The basic UNITY theory (revised version, based upon the "co" operator)
     6 The basic UNITY theory (revised version, based upon the "co" operator)
     7 
     7 
     8 From Misra, "A Logic for Concurrent Programming", 1994
     8 From Misra, "A Logic for Concurrent Programming", 1994
     9 *)
     9 *)
    10 
    10 
    11 UNITY = LessThan + ListOrder +
    11 UNITY = Main + 
    12 
       
    13 
    12 
    14 typedef (Program)
    13 typedef (Program)
    15   'a program = "{(init:: 'a set, acts :: ('a * 'a)set set). Id:acts}"
    14   'a program = "{(init:: 'a set, acts :: ('a * 'a)set set). Id:acts}"
    16 
    15 
    17 consts
    16 consts