1
2
FOL = IFOL +
3
4
rules
5
classical "(~P ==> P) ==> P"
6
7
end
8
9
ML val thy_data = [ClasetThyData.thy_data];