src/HOL/Lambda/InductTermi.thy
changeset 5261 ce3c25c8a694
child 5717 0d28dbe484b6
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Lambda/InductTermi.thy	Thu Aug 06 10:33:54 1998 +0200
@@ -0,0 +1,22 @@
+(*  Title:      HOL/Lambda/InductTermi.thy
+    ID:         $Id$
+    Author:     Tobias Nipkow
+    Copyright   1998 TU Muenchen
+
+Inductive characterization of terminating lambda terms.
+Goes back to
+Raamsdonk & Severi. On normalization. CWI TR CS-R9545, 1995.
+Also rediscovered by Matthes and Joachimski.
+*)
+
+InductTermi = Acc + ListBeta +
+
+consts IT :: dB set
+inductive IT
+intrs
+VarI "rs : lists IT ==> (Var n)$$rs : IT"
+LambdaI "r : IT ==> Abs r : IT"
+BetaI "[| (r[s/0])$$ss : IT; s : IT |] ==> (Abs r $ s)$$ss : IT"
+monos "[lists_mono]"
+
+end