merged
authornipkow
Wed, 02 Oct 2013 23:05:36 +0200
changeset 54048 f6bd38fb2c39
parent 54046 16374631b504 (current diff)
parent 54047 83fb090dae9e (diff)
child 54049 566b769c3477
merged
--- a/src/HOL/Library/While_Combinator.thy	Wed Oct 02 22:59:54 2013 +0200
+++ b/src/HOL/Library/While_Combinator.thy	Wed Oct 02 23:05:36 2013 +0200
@@ -1,7 +1,6 @@
 (*  Title:      HOL/Library/While_Combinator.thy
     Author:     Tobias Nipkow
     Author:     Alexander Krauss
-    Copyright   2000 TU Muenchen
 *)
 
 header {* A general ``while'' combinator *}
@@ -257,7 +256,7 @@
   while_option (%(ws,_). ws \<noteq> [] \<and> p(hd ws))
     ((%(ws,Z).
      let x = hd ws; new = filter (\<lambda>y. y \<notin> Z) (f x)
-     in (new @ tl ws, set new \<union> insert x Z)))
+     in (new @ tl ws, set new \<union> Z)))
     ([x],{x})"
 
 lemma rtrancl_while_Some: assumes "rtrancl_while p f x = Some(ws,Z)"
@@ -268,7 +267,7 @@
   let ?test = "(%(ws,_). ws \<noteq> [] \<and> p(hd ws))"
   let ?step = "(%(ws,Z).
      let x = hd ws; new = filter (\<lambda>y. y \<notin> Z) (f x)
-     in (new @ tl ws, set new \<union> insert x Z))"
+     in (new @ tl ws, set new \<union> Z))"
   let ?R = "{(x,y). y \<in> set(f x)}"
   let ?Inv = "%(ws,Z). x \<in> Z \<and> set ws \<subseteq> Z \<and> ?R `` (Z - set ws) \<subseteq> Z \<and>
                        Z \<subseteq> ?R^* `` {x} \<and> (\<forall>z\<in>Z - set ws. p z)"