src/HOLCF/FOCUS/Stream_adm.thy
changeset 11350 4c55b020d6ee
child 11355 778c369559d9
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOLCF/FOCUS/Stream_adm.thy	Thu May 31 16:53:00 2001 +0200
@@ -0,0 +1,29 @@
+(*  Title: 	HOLCF/ex/Stream_adm.thy
+    ID:         $ $
+    Author: 	David von Oheimb, TU Muenchen
+    License:    GPL (GNU GENERAL PUBLIC LICENSE)
+
+Admissibility for streams
+*)
+
+Stream_adm = Stream + Continuity +
+
+consts
+
+  stream_monoP,
+  stream_antiP	:: "(('a stream) set \\<Rightarrow> ('a stream) set) \\<Rightarrow> bool"
+
+defs
+
+  stream_monoP_def "stream_monoP F \\<equiv> \\<exists>Q i. \\<forall>P s. Fin i \\<le> #s \\<longrightarrow> 
+			s \\<in> F P = (stream_take i\\<cdot>s \\<in> Q \\<and> iterate i rt s \\<in> P)"
+  stream_antiP_def "stream_antiP F \\<equiv> \\<forall>P x. \\<exists>Q i. 
+		(#x  < Fin i \\<longrightarrow> (\\<forall>y. x \\<sqsubseteq> y \\<longrightarrow> y \\<in> F P \\<longrightarrow> x \\<in> F P)) \\<and>
+		(Fin i <= #x \\<longrightarrow> (\\<forall>y. x \\<sqsubseteq> y \\<longrightarrow> 
+		y \\<in> F P = (stream_take i\\<cdot>y \\<in> Q \\<and> iterate i rt y \\<in> P)))"
+
+constdefs
+  antitonP :: "'a set => bool"
+ "antitonP P \\<equiv> \\<forall>x y. x \\<sqsubseteq> y \\<longrightarrow> y\\<in>P \\<longrightarrow> x\\<in>P"
+  
+end