QuotTest.thy
changeset 254 77ff9624cfd6
parent 230 84a356e3d38b
child 284 78bc4d9d7975
equal deleted inserted replaced
252:e30997c88050 254:77ff9624cfd6
     1 theory QuotTest
     1 theory QuotTest
     2 imports QuotMain
     2 imports QuotMain
     3 begin
     3 begin
       
     4 
     4 
     5 
     5 section {* various tests for quotient types*}
     6 section {* various tests for quotient types*}
     6 datatype trm =
     7 datatype trm =
     7   var  "nat"
     8   var  "nat"
     8 | app  "trm" "trm"
     9 | app  "trm" "trm"