src/ZF/Induct/ListN.thy
changeset 12088 6f463d16cbd0
child 12560 5820841f21fd
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/ZF/Induct/ListN.thy	Wed Nov 07 12:29:07 2001 +0100
@@ -0,0 +1,22 @@
+(*  Title:      ZF/ex/ListN
+    ID:         $Id$
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
+    Copyright   1994  University of Cambridge
+
+Inductive definition of lists of n elements
+
+See Ch. Paulin-Mohring, Inductive Definitions in the System Coq.
+Research Report 92-49, LIP, ENS Lyon.  Dec 1992.
+*)
+
+ListN = Main +
+
+consts  listn ::i=>i
+inductive
+  domains   "listn(A)" <= "nat*list(A)"
+  intrs
+    NilI  "<0,Nil> \\<in> listn(A)"
+    ConsI "[| a \\<in> A; <n,l> \\<in> listn(A) |] ==> <succ(n), Cons(a,l)> \\<in> listn(A)"
+  type_intrs "nat_typechecks @ list.intrs"
+
+end