src/HOL/Library/Rewrite.thy
author wenzelm
Sun, 29 Mar 2015 19:32:27 +0200
changeset 59842 9fda99b3d5ee
parent 59739 4ed50ebf5d36
child 59975 da10875adf8e
permissions -rw-r--r--
tuned;

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