src/HOL/Library/Rewrite.thy
changeset 60047 58e5b16cbd94
parent 59975 da10875adf8e
child 60054 ef4878146485
equal deleted inserted replaced
60042:7ff7fdfbb9a0 60047:58e5b16cbd94
     8 imports Main
     8 imports Main
     9 begin
     9 begin
    10 
    10 
    11 consts rewrite_HOLE :: "'a::{}"
    11 consts rewrite_HOLE :: "'a::{}"
    12 notation rewrite_HOLE ("HOLE")
    12 notation rewrite_HOLE ("HOLE")
    13 notation rewrite_HOLE ("\<box>")
    13 notation rewrite_HOLE ("\<hole>")
    14 
    14 
    15 lemma eta_expand:
    15 lemma eta_expand:
    16   fixes f :: "'a::{} \<Rightarrow> 'b::{}"
    16   fixes f :: "'a::{} \<Rightarrow> 'b::{}"
    17   shows "f \<equiv> \<lambda>x. f x" .
    17   shows "f \<equiv> \<lambda>x. f x" .
    18 
    18