author | wenzelm |
Wed, 08 Apr 2015 21:24:27 +0200 | |
changeset 59975 | da10875adf8e |
parent 59739 | 4ed50ebf5d36 |
child 60047 | 58e5b16cbd94 |
permissions | -rw-r--r-- |
(* Title: HOL/Library/Rewrite.thy Author: Christoph Traut, Lars Noschinski, TU Muenchen Proof method "rewrite" with support for subterm-selection based on patterns. *) 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" . ML_file "cconv.ML" ML_file "rewrite.ML" end