# HG changeset patch # User Andreas Lochbihler # Date 1447689732 -3600 # Node ID 7ba83fbac0ae3ad58e556c97e7d3cda7affbf72e # Parent d04b1b4fb01548d425f1d7a24d871e4275cd0ed9# Parent e4d7972402ed764147837796559135e9e851e403 merged diff -r d04b1b4fb015 -r 7ba83fbac0ae src/HOL/Complete_Partial_Order.thy --- a/src/HOL/Complete_Partial_Order.thy Mon Nov 16 15:59:47 2015 +0100 +++ b/src/HOL/Complete_Partial_Order.thy Mon Nov 16 17:02:12 2015 +0100 @@ -87,12 +87,16 @@ subsection \Transfinite iteration of a function\ +context notes [[inductive_defs]] begin + inductive_set iterates :: "('a \ 'a) \ 'a set" for f :: "'a \ 'a" where step: "x \ iterates f \ f x \ iterates f" | Sup: "chain (op \) M \ \x\M. x \ iterates f \ Sup M \ iterates f" +end + lemma iterates_le_f: "x \ iterates f \ monotone (op \) (op \) f \ x \ f x" by (induct x rule: iterates.induct)