src/HOLCF/IOA/meta_theory/Seq.thy
changeset 5102 8c782c25a11e
parent 4283 92707e24b62b
child 5976 44290b71a85f
--- a/src/HOLCF/IOA/meta_theory/Seq.thy	Tue Jun 30 20:50:34 1998 +0200
+++ b/src/HOLCF/IOA/meta_theory/Seq.thy	Tue Jun 30 20:51:15 1998 +0200
@@ -7,7 +7,7 @@
 *)  
 
 
-Seq = HOLCF + 
+Seq = HOLCF + Inductive +
 
 domain 'a seq = nil | "##" (HD::'a) (lazy TL::'a seq)  (infixr 65)