src/FOLP/FOLP.thy
author lcp
Wed, 03 May 1995 17:38:27 +0200
changeset 1105 136b05aa77ed
parent 0 a5a9c433f639
child 1142 eb0e2ff8f032
permissions -rw-r--r--
Modified proofs for (q)split, fst, snd for new definitions. The rule f(q)splitE is now called (q)splitE and is weaker than before. The rule '(q)split' is now a meta-equality; this required modifying all proofs involving e.g. split RS trans.

FOLP = IFOLP +
consts
  cla :: "[p=>p]=>p"
rules
  classical "(!!x.x:~P ==> f(x):P) ==> cla(f):P"
end