src/HOL/Lambda/InductTermi.thy
changeset 5261 ce3c25c8a694
child 5717 0d28dbe484b6
equal deleted inserted replaced
5260:1835a591d3a7 5261:ce3c25c8a694
       
     1 (*  Title:      HOL/Lambda/InductTermi.thy
       
     2     ID:         $Id$
       
     3     Author:     Tobias Nipkow
       
     4     Copyright   1998 TU Muenchen
       
     5 
       
     6 Inductive characterization of terminating lambda terms.
       
     7 Goes back to
       
     8 Raamsdonk & Severi. On normalization. CWI TR CS-R9545, 1995.
       
     9 Also rediscovered by Matthes and Joachimski.
       
    10 *)
       
    11 
       
    12 InductTermi = Acc + ListBeta +
       
    13 
       
    14 consts IT :: dB set
       
    15 inductive IT
       
    16 intrs
       
    17 VarI "rs : lists IT ==> (Var n)$$rs : IT"
       
    18 LambdaI "r : IT ==> Abs r : IT"
       
    19 BetaI "[| (r[s/0])$$ss : IT; s : IT |] ==> (Abs r $ s)$$ss : IT"
       
    20 monos "[lists_mono]"
       
    21 
       
    22 end