src/ZF/ex/Ntree.thy
changeset 515 abcc438e7c27
child 539 01906e4644e0
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/ZF/ex/Ntree.thy	Fri Aug 12 12:28:46 1994 +0200
@@ -0,0 +1,23 @@
+(*  Title: 	ZF/ex/Ntree.ML
+    ID:         $Id$
+    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Copyright   1994  University of Cambridge
+
+Datatype definition n-ary branching trees
+Demonstrates a simple use of function space in a datatype definition
+   and also "nested" monotonicity theorems
+
+Based upon ex/Term.thy
+*)
+
+Ntree = InfDatatype +
+consts
+  ntree :: "i=>i"
+
+datatype
+  "ntree(A)" = Branch ("a: A", "h: (UN n:nat. n -> ntree(A))")
+  monos	      "[[subset_refl, Pi_mono] MRS UN_mono]"
+  type_intrs  "[nat_fun_univ RS subsetD]"
+  type_elims  "[UN_E]"
+
+end