diff -r 97a8ff4e4ac9 -r c8cc5ab4a863 src/HOL/ATP.thy --- a/src/HOL/ATP.thy Fri Oct 18 10:43:20 2013 +0200 +++ b/src/HOL/ATP.thy Fri Oct 18 10:43:21 2013 +0200 @@ -18,34 +18,34 @@ subsection {* Higher-order reasoning helpers *} -definition fFalse :: bool where [no_atp]: +definition fFalse :: bool where "fFalse \ False" -definition fTrue :: bool where [no_atp]: +definition fTrue :: bool where "fTrue \ True" -definition fNot :: "bool \ bool" where [no_atp]: +definition fNot :: "bool \ bool" where "fNot P \ \ P" -definition fComp :: "('a \ bool) \ 'a \ bool" where [no_atp]: +definition fComp :: "('a \ bool) \ 'a \ bool" where "fComp P = (\x. \ P x)" -definition fconj :: "bool \ bool \ bool" where [no_atp]: +definition fconj :: "bool \ bool \ bool" where "fconj P Q \ P \ Q" -definition fdisj :: "bool \ bool \ bool" where [no_atp]: +definition fdisj :: "bool \ bool \ bool" where "fdisj P Q \ P \ Q" -definition fimplies :: "bool \ bool \ bool" where [no_atp]: +definition fimplies :: "bool \ bool \ bool" where "fimplies P Q \ (P \ Q)" -definition fequal :: "'a \ 'a \ bool" where [no_atp]: +definition fequal :: "'a \ 'a \ bool" where "fequal x y \ (x = y)" -definition fAll :: "('a \ bool) \ bool" where [no_atp]: +definition fAll :: "('a \ bool) \ bool" where "fAll P \ All P" -definition fEx :: "('a \ bool) \ bool" where [no_atp]: +definition fEx :: "('a \ bool) \ bool" where "fEx P \ Ex P" lemma fTrue_ne_fFalse: "fFalse \ fTrue"