diff -r a3d2a6b6693e -r 0d28dbe484b6 src/HOL/Induct/Term.thy --- a/src/HOL/Induct/Term.thy Wed Oct 21 17:46:00 1998 +0200 +++ b/src/HOL/Induct/Term.thy Wed Oct 21 17:48:02 1998 +0200 @@ -28,7 +28,7 @@ inductive "term(A)" intrs APP_I "[| M: A; N : list(term(A)) |] ==> Scons M N : term(A)" - monos "[list_mono]" + monos list_mono defs (*defining abstraction/representation functions for term list...*)