author | noschinl |
Wed, 18 Mar 2015 13:51:33 +0100 | |
changeset 59739 | 4ed50ebf5d36 |
child 59975 | da10875adf8e |
permissions | -rw-r--r-- |
theory Rewrite imports Main begin consts rewrite_HOLE :: "'a :: {}" notation rewrite_HOLE ("HOLE") notation rewrite_HOLE ("\<box>") lemma eta_expand: fixes f :: "'a :: {} \<Rightarrow> 'b :: {}" shows "f \<equiv> (\<lambda>x. f x)" by (rule reflexive) ML_file "cconv.ML" ML_file "rewrite.ML" setup Rewrite.setup end