diff -r 97a8ff4e4ac9 -r c8cc5ab4a863 src/HOL/Metis.thy --- a/src/HOL/Metis.thy Fri Oct 18 10:43:20 2013 +0200 +++ b/src/HOL/Metis.thy Fri Oct 18 10:43:21 2013 +0200 @@ -16,7 +16,7 @@ subsection {* Literal selection and lambda-lifting helpers *} definition select :: "'a \ 'a" where -[no_atp]: "select = (\x. x)" +"select = (\x. x)" lemma not_atomize: "(\ A \ False) \ Trueprop A" by (cut_tac atomize_not [of "\ A"]) simp @@ -30,7 +30,7 @@ lemma select_FalseI: "False \ select False" by simp definition lambda :: "'a \ 'a" where -[no_atp]: "lambda = (\x. x)" +"lambda = (\x. x)" lemma eq_lambdaI: "x \ y \ x \ lambda y" unfolding lambda_def by assumption