src/HOL/Proofs/Lambda/WeakNorm.thy
changeset 41413 64cd30d6b0b8
parent 40627 becf5d5187cc
child 42364 8c674b3b8e44
equal deleted inserted replaced
41412:35f30e07fe0d 41413:64cd30d6b0b8
     4 *)
     4 *)
     5 
     5 
     6 header {* Weak normalization for simply-typed lambda calculus *}
     6 header {* Weak normalization for simply-typed lambda calculus *}
     7 
     7 
     8 theory WeakNorm
     8 theory WeakNorm
     9 imports Type NormalForm Code_Integer
     9 imports Type NormalForm "~~/src/HOL/Library/Code_Integer"
    10 begin
    10 begin
    11 
    11 
    12 text {*
    12 text {*
    13 Formalization by Stefan Berghofer. Partly based on a paper proof by
    13 Formalization by Stefan Berghofer. Partly based on a paper proof by
    14 Felix Joachimski and Ralph Matthes \cite{Matthes-Joachimski-AML}.
    14 Felix Joachimski and Ralph Matthes \cite{Matthes-Joachimski-AML}.