Nominal/Ex/Test.thy
changeset 1795 e39453c8b186
parent 1773 c0eac04ae3b4
child 2045 6800fcaafa2a
equal deleted inserted replaced
1794:d51aab59bfbf 1795:e39453c8b186
     1 (*<*)
       
     2 theory Test
     1 theory Test
     3 imports "../Parser"
     2 imports "../Parser"
     4 begin
     3 begin
     5 
     4 
     6 (* This file contains only the examples that are not supposed to work yet. *)
     5 (* This file contains only the examples that are not supposed to work yet. *)
    36 where
    35 where
    37   "bv8 (Bar0 x) = {}"
    36   "bv8 (Bar0 x) = {}"
    38 | "bv8 (Bar1 v x b) = {atom v}"
    37 | "bv8 (Bar1 v x b) = {atom v}"
    39 *)
    38 *)
    40 
    39 
    41 (* example 9 from Peter Sewell's bestiary *)
       
    42 (* run out of steam at the moment *)
       
    43 
       
    44 end
    40 end
    45 (*>*)
       
    46 
    41 
    47 
    42