src/FOLP/FOLP.thy
changeset 0 a5a9c433f639
child 1142 eb0e2ff8f032
equal deleted inserted replaced
-1:000000000000 0:a5a9c433f639
       
     1 FOLP = IFOLP +
       
     2 consts
       
     3   cla :: "[p=>p]=>p"
       
     4 rules
       
     5   classical "(!!x.x:~P ==> f(x):P) ==> cla(f):P"
       
     6 end