src/HOL/Auth/NS_Public.thy
changeset 2549 0c723635b9e6
parent 2538 c55f68761a8d
child 3465 e85c24717cad
equal deleted inserted replaced
2548:b5d19d99a58d 2549:0c723635b9e6
     7 Version incorporating Lowe's fix (inclusion of B's identity in round 2).
     7 Version incorporating Lowe's fix (inclusion of B's identity in round 2).
     8 *)
     8 *)
     9 
     9 
    10 NS_Public = Public + 
    10 NS_Public = Public + 
    11 
    11 
    12 consts  lost    :: agent set        (*No need for it to be a variable*)
    12 consts  lost       :: agent set        (*No need for it to be a variable*)
    13 	ns_public  :: event list set
    13 	ns_public  :: event list set
       
    14 
    14 inductive ns_public
    15 inductive ns_public
    15   intrs 
    16   intrs 
    16          (*Initial trace is empty*)
    17          (*Initial trace is empty*)
    17     Nil  "[]: ns_public"
    18     Nil  "[]: ns_public"
    18 
    19