Loading theory "HOL-Analysis.L2_Norm" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space" via "HOL-Analysis.Linear_Algebra" via "HOL-Analysis.Euclidean_Space") Loading theory "HOL-Analysis.Inner_Product" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space" via "HOL-Analysis.Linear_Algebra" via "HOL-Analysis.Euclidean_Space" via "HOL-Analysis.Product_Vector") ### theory "HOL-Analysis.L2_Norm" ### 0.251s elapsed time, 0.572s cpu time, 0.000s GC time Loading theory "HOL-Analysis.Norm_Arith" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space") class real_inner = dist_norm + real_vector + sgn_div_norm + uniformity_dist + open_uniformity + fixes inner :: "'a \ 'a \ real" assumes "inner_commute": "\x y. inner x y = inner y x" and "inner_add_left": "\x y z. inner (x + y) z = inner x z + inner y z" and "inner_scaleR_left": "\r x y. inner (r *\<^sub>R x) y = r * inner x y" and "inner_ge_zero": "\x. 0 \ inner x x" and "inner_eq_zero_iff": "\x. (inner x x = 0) = (x = (0::'a))" and "norm_eq_sqrt_inner": "\x. norm x = sqrt (inner x x)" ### ML warning (line 103 of "~~/src/HOL/Analysis/normarith.ML"): ### Matches are not exhaustive. ### ML warning (line 347 of "~~/src/HOL/Analysis/normarith.ML"): ### Value identifier (instantiate_cterm') has not been referenced. signature NORM_ARITH = sig val norm_arith: Proof.context -> conv val norm_arith_tac: Proof.context -> int -> tactic end structure NormArith: NORM_ARITH ### theory "HOL-Analysis.Norm_Arith" ### 0.425s elapsed time, 0.848s cpu time, 0.000s GC time instantiation real :: real_inner inner_real == inner :: real \ real \ real instantiation complex :: real_inner inner_complex == inner :: complex \ complex \ real ### theory "HOL-Analysis.Inner_Product" ### 1.401s elapsed time, 2.872s cpu time, 0.000s GC time Loading theory "HOL-Analysis.Product_Vector" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space" via "HOL-Analysis.Linear_Algebra" via "HOL-Analysis.Euclidean_Space") instantiation prod :: (real_vector, real_vector) real_vector scaleR_prod == scaleR :: real \ 'a \ 'b \ 'a \ 'b instantiation prod :: (metric_space, metric_space) dist dist_prod == dist :: 'a \ 'b \ 'a \ 'b \ real instantiation prod :: (metric_space, metric_space) uniformity_dist uniformity_prod == uniformity :: (('a \ 'b) \ 'a \ 'b) filter instantiation prod :: (metric_space, metric_space) metric_space instantiation prod :: (real_normed_vector, real_normed_vector) real_normed_vector sgn_prod == sgn :: 'a \ 'b \ 'a \ 'b norm_prod == norm :: 'a \ 'b \ real instantiation prod :: (real_inner, real_inner) real_inner inner_prod == inner :: 'a \ 'b \ 'a \ 'b \ real ### theory "HOL-Analysis.Product_Vector" ### 0.726s elapsed time, 1.408s cpu time, 0.180s GC time Loading theory "HOL-Analysis.Euclidean_Space" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space" via "HOL-Analysis.Linear_Algebra") class euclidean_space = real_inner + fixes Basis :: "'a set" assumes "nonempty_Basis": "Basis \ {}" assumes "finite_Basis": "finite Basis" assumes "inner_Basis": "\u v. \u \ Basis; v \ Basis\ \ inner u v = (if u = v then 1 else 0)" assumes "euclidean_all_zero_iff": "\x. (\u\Basis. inner x u = 0) = (x = (0::'a))" instantiation real :: euclidean_space Basis_real == Basis :: real set instantiation complex :: euclidean_space Basis_complex == Basis :: complex set instantiation prod :: (euclidean_space, euclidean_space) euclidean_space Basis_prod == Basis :: ('a \ 'b) set ### theory "HOL-Analysis.Euclidean_Space" ### 1.876s elapsed time, 2.536s cpu time, 0.000s GC time Loading theory "HOL-Analysis.Linear_Algebra" (required by "HOL-Analysis.Extended_Real_Limits" via "HOL-Analysis.Topology_Euclidean_Space") Proofs for inductive predicate(s) "span_induct_alt_helpp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the induction rule ... Proving the simplification rules ... class real_inner = real_normed_vector + fixes inner :: "'a \ 'a \ real" assumes "inner_commute": "\x y. x \ y = y \ x" and "inner_add_left": "\x y z. (x + y) \ z = x \ z + y \ z" and "inner_scaleR_left": "\r x y. r *\<^sub>R x \ y = r * (x \ y)" and "inner_ge_zero": "\x. 0 \ x \ x" and "inner_eq_zero_iff": "\x. (x \ x = 0) = (x = (0::'a))" and "norm_eq_sqrt_inner": "\x. norm x = sqrt (x \ x)" ### theory "HOL-Analysis.Linear_Algebra" ### 3.673s elapsed time, 6.708s cpu time, 0.460s GC time Loading theory "HOL-Analysis.Topology_Euclidean_Space" (required by "HOL-Analysis.Extended_Real_Limits") class topological_space = open + assumes "open_UNIV": "open UNIV" assumes "open_Int": "\S T. \open S; open T\ \ open (S \ T)" assumes "open_Union": "\K. Ball K open \ open (\K)" locale countable_basis fixes B :: "'a set set" assumes "countable_basis B" class second_countable_topology = topological_space + assumes "ex_countable_subbasis": "\B. countable B \ open = generate_topology B" ### Ignoring duplicate rewrite rule: ### span UNIV \ UNIV ### Ignoring duplicate rewrite rule: ### span UNIV \ UNIV ### Ignoring duplicate rewrite rule: ### of_nat (Suc ?m1) \ (1::?'a1) + of_nat ?m1 class heine_borel = metric_space + assumes "bounded_imp_convergent_subsequence": "\f. bounded (range f) \ \l r. strict_mono r \ (f \ r) \ l" ### Ignoring duplicate rewrite rule: ### dim (span ?S1) \ dim ?S1 ### Ignoring duplicate rewrite rule: ### dim (span ?S1) \ dim ?S1 ### Ignoring duplicate rewrite rule: ### dim (span ?S1) \ dim ?S1 ### Ignoring duplicate rewrite rule: ### dim UNIV \ DIM(?'a1) ### Ignoring duplicate rewrite rule: ### (0::?'a1) \ span ?S1 \ True ### Ignoring duplicate rewrite rule: ### (0::?'a1) \ span ?S1 \ True ### theory "HOL-Analysis.Topology_Euclidean_Space" ### 8.176s elapsed time, 16.328s cpu time, 0.872s GC time Loading theory "HOL-Analysis.Extended_Real_Limits" ### Ignoring duplicate rewrite rule: ### collinear {?x1, ?y1} \ True ### theory "HOL-Analysis.Extended_Real_Limits" ### 1.590s elapsed time, 3.164s cpu time, 0.344s GC time ### Rule already declared as introduction (intro) ### \finite ?S; \T\?S. open T\ ### \ open (\?S) ### Ignoring duplicate rewrite rule: ### ?y1 \ ball ?x1 ?e1 \ dist ?x1 ?y1 < ?e1 ### Ignoring duplicate rewrite rule: ### 0 < DIM(?'a1) \ True ### Ignoring duplicate rewrite rule: ### 0 < dist ?x1 ?y1 \ ?x1 \ ?y1 ### Ignoring duplicate introduction (intro) ### ((\x. x) \ ?a) (at ?a within ?s) ### Ignoring duplicate introduction (intro) ### ((\x. ?k) \ ?k) ?F ### Ignoring duplicate introduction (intro) ### ((\x. x) \ ?a) (at ?a within ?s) ### Ignoring duplicate introduction (intro) ### ((\x. ?k) \ ?k) ?F ### Ignoring duplicate introduction (intro) ### ((\x. x) \ ?a) (at ?a within ?s) ### Ignoring duplicate introduction (intro) ### ((\x. ?k) \ ?k) ?F ### Ignoring duplicate introduction (intro) ### ((\x. x) \ ?a) (at ?a within ?s) ### Ignoring duplicate introduction (intro) ### ((\x. ?k) \ ?k) ?F ### Ignoring duplicate rewrite rule: ### sup ?x1 (- ?x1) \ top ### Rule already declared as introduction (intro) ### countable ?A \ countable (?f ` ?A) ### Rule already declared as introduction (intro) ### \countable ?I; ### \i. i \ ?I \ countable (?A i)\ ### \ countable (Sigma ?I ?A) ### Rule already declared as introduction (intro) ### \countable ?I; ### \i. i \ ?I \ countable (?A i)\ ### \ countable (\i\?I. ?A i) ### Ignoring duplicate rewrite rule: ### 0 < DIM(?'a1) \ True ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Ignoring duplicate rewrite rule: ### of_nat (Suc ?m1) \ (1::?'a1) + of_nat ?m1 ### Metis: Unused theorems: "Real_Vector_Spaces.metric_space_class.dist_nz" ### Ignoring duplicate rewrite rule: ### 0 < dist ?x1 ?y1 \ ?x1 \ ?y1 ### Ignoring duplicate rewrite rule: ### 0 < dist ?x1 ?y1 \ ?x1 \ ?y1 Loading theory "Coinductive.Resumption" (required by "Coinductive.Coinductive_Examples") Loading theory "Coinductive.Coinductive_Nat" (required by "Coinductive.Coinductive" via "Coinductive.Coinductive_List_Prefix" via "Coinductive.Coinductive_List") Proofs for coinductive predicate(s) "resumptionp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... Proofs for coinductive predicate(s) "enat_setp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... locale co Proofs for coinductive predicate(s) "Le_enatp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... ### theory "Coinductive.Coinductive_Nat" ### 1.060s elapsed time, 2.168s cpu time, 0.000s GC time Loading theory "Coinductive.Coinductive_List" (required by "Coinductive.Coinductive" via "Coinductive.Coinductive_List_Prefix") consts RESUMPTION_corec_aux :: "nat \ ('e \ ('a, 'b, 'c, 'd, 'e) resumption_corec) \ 'e \ ('c + 'b + 'a, 'd) Old_Datatype.node set" Proofs for coinductive predicate(s) "Eq_RESUMPTION" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... ### theory "Coinductive.Resumption" ### 1.306s elapsed time, 2.672s cpu time, 0.000s GC time Loading theory "Coinductive.CCPO_Topology" (required by "Coinductive.Coinductive_Examples" via "Coinductive.LList_CCPO_Topology") class ccpo_topology = ccpo + open + assumes "open_ccpo": "\A. open A = (\C. chain C \ C \ {} \ \C \ A \ C \ A \ {})" consts unfold_llist :: "('a \ bool) \ ('a \ 'b) \ ('a \ 'a) \ 'a \ 'b llist" Proofs for inductive predicate(s) "lsetp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the induction rule ... Proving the simplification rules ... Proofs for inductive predicate(s) "lfinite" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the induction rule ... Proving the simplification rules ... consts lappend :: "'a llist \ 'a llist \ 'a llist" ### Ignoring duplicate rewrite rule: ### lnull (lappend ?xs1 ?ys1) \ lnull ?xs1 \ lnull ?ys1 Proofs for coinductive predicate(s) "lprefix" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... consts lSup :: "'a llist set \ 'a llist" instantiation set :: (type) ccpo_topology open_set == open :: 'a set set \ bool instantiation enat :: ccpo_topology ### theory "Coinductive.CCPO_Topology" ### 2.346s elapsed time, 4.656s cpu time, 0.412s GC time consts iterates :: "('a \ 'a) \ 'a \ 'a llist" consts llist_of :: "'a list \ 'a llist" consts ltake :: "enat \ 'a llist \ 'a llist" ### Ambiguous input (line 1018 of "~~/afp/thys/Coinductive/Coinductive_List.thy") produces 2 parse trees: ### ("\<^const>HOL.Trueprop" ### ("\<^const>HOL.eq" ### ("_applC" ("_position" ldrop) ### ("_cargs" ("_position" n) ("_position" xs))) ### ("_case_syntax" ("_position" n) ### ("_case2" ### ("_case1" ("\<^const>Groups.zero_class.zero") ("_position" xs)) ### ("_case2" ### ("_case1" ("_applC" ("_position" eSuc) ("_position" n')) ### ("_case_syntax" ("_position" xs) ### ("_case1" ("_position" LNil) ("_position" LNil)))) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_applC" ("_position" ldrop) ### ("_cargs" ("_position" n') ("_position" xs'))))))))) ### ("\<^const>HOL.Trueprop" ### ("\<^const>HOL.eq" ### ("_applC" ("_position" ldrop) ### ("_cargs" ("_position" n) ("_position" xs))) ### ("_case_syntax" ("_position" n) ### ("_case2" ### ("_case1" ("\<^const>Groups.zero_class.zero") ("_position" xs)) ### ("_case1" ("_applC" ("_position" eSuc) ("_position" n')) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_applC" ("_position" ldrop) ### ("_cargs" ("_position" n') ("_position" xs'))))))))))) ### Fortunately, only one parse tree is well-formed and type-correct, ### but you may still want to disambiguate your grammar or your input. consts ltakeWhile :: "('a \ bool) \ 'a llist \ 'a llist" consts lnth :: "'a llist \ nat \ 'a" consts lzip :: "'a llist \ 'b llist \ ('a \ 'b) llist" Proofs for coinductive predicate(s) "ldistinct" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... Proofs for coinductive predicate(s) "llexord" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... ### Ambiguous input (line 1491 of "~~/afp/thys/Coinductive/Coinductive_List.thy") produces 2 parse trees: ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" ltake) ### ("_pttrns" ("_position" n) ("_position" xs))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs))) ### ("_case_syntax" ("_position" n) ### ("_case2" ### ("_case1" ("\<^const>Groups.zero_class.zero") ### ("_position" LNil)) ### ("_case1" ("_applC" ("_position" eSuc) ("_position" n)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" ltake) ### ("_cargs" ("_position" n) ("_position" xs))))))))))))) ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" ltake) ### ("_pttrns" ("_position" n) ("_position" xs))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case2" ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs))) ### ("_case_syntax" ("_position" n) ### ("_case1" ("\<^const>Groups.zero_class.zero") ### ("_position" LNil)))) ### ("_case1" ("_applC" ("_position" eSuc) ("_position" n)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" ltake) ### ("_cargs" ("_position" n) ("_position" xs))))))))))) ### Fortunately, only one parse tree is well-formed and type-correct, ### but you may still want to disambiguate your grammar or your input. ### Ignoring duplicate rewrite rule: ### lnull (lzip ?xs1 ?ys1) \ lnull ?xs1 \ lnull ?ys1 ### Ambiguous input (line 2468 of "~~/afp/thys/Coinductive/Coinductive_List.thy") produces 2 parse trees: ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" lzip) ### ("_pattern" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("_applC" ("_position" LCons) ### ("_cargs" ### ("_tuple" ("_position" x) ### ("_tuple_arg" ("_position" y))) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lzip) ### ("_cargs" ("_position" xs') ### ("_position" ys')))))))))))))) ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" lzip) ### ("_pattern" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case2" ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case1" ("_position" LNil) ("_position" LNil)))) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("_applC" ("_position" LCons) ### ("_cargs" ### ("_tuple" ("_position" x) ("_tuple_arg" ("_position" y))) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lzip) ### ("_cargs" ("_position" xs') ("_position" ys')))))))))))) ### Fortunately, only one parse tree is well-formed and type-correct, ### but you may still want to disambiguate your grammar or your input. class ord = type + fixes less_eq :: "'a \ 'a \ bool" and less :: "'a \ 'a \ bool" Proofs for coinductive predicate(s) "lsorted" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... ### Partially applied constant "Sublist.list_emb" on left hand side of equation, in theorem: ### subseq_order.lsorted LNil \ True ### Partially applied constant "Sublist.list_emb" on left hand side of equation, in theorem: ### subseq_order.lsorted (LCons ?x LNil) \ True ### Partially applied constant "Sublist.list_emb" on left hand side of equation, in theorem: ### subseq_order.lsorted (LCons ?x (LCons ?y ?xs)) \ ### subseq ?x ?y \ subseq_order.lsorted (LCons ?y ?xs) ### Partially applied constant "Sublist.sublist" on left hand side of equation, in theorem: ### sublist_order.lsorted LNil \ True ### Partially applied constant "Sublist.sublist" on left hand side of equation, in theorem: ### sublist_order.lsorted (LCons ?x LNil) \ True ### Partially applied constant "Sublist.sublist" on left hand side of equation, in theorem: ### sublist_order.lsorted (LCons ?x (LCons ?y ?xs)) \ ### sublist ?x ?y \ sublist_order.lsorted (LCons ?y ?xs) ### Partially applied constant "Sublist.suffix" on left hand side of equation, in theorem: ### suffix_order.lsorted LNil \ True ### Partially applied constant "Sublist.suffix" on left hand side of equation, in theorem: ### suffix_order.lsorted (LCons ?x LNil) \ True ### Partially applied constant "Sublist.suffix" on left hand side of equation, in theorem: ### suffix_order.lsorted (LCons ?x (LCons ?y ?xs)) \ ### suffix ?x ?y \ suffix_order.lsorted (LCons ?y ?xs) ### Partially applied constant "Sublist.prefix" on left hand side of equation, in theorem: ### prefix_order.lsorted LNil \ True ### Partially applied constant "Sublist.prefix" on left hand side of equation, in theorem: ### prefix_order.lsorted (LCons ?x LNil) \ True ### Partially applied constant "Sublist.prefix" on left hand side of equation, in theorem: ### prefix_order.lsorted (LCons ?x (LCons ?y ?xs)) \ ### prefix ?x ?y \ prefix_order.lsorted (LCons ?y ?xs) class preorder = ord + assumes "less_le_not_le": "\x y. (x < y) = (x \ y \ \ y \ x)" and "order_refl": "\x. x \ x" and "order_trans": "\x y z. \x \ y; y \ z\ \ x \ z" class linorder = order + assumes "linear": "\x y. x \ y \ y \ x" ### Legacy feature! Old 'def' command -- use 'define' instead ### Introduced fixed type variable(s): 'a in "P__" or "xs__" ### Legacy feature! Old 'def' command -- use 'define' instead ### Introduced fixed type variable(s): 'a in "P__" or "xs__" ### Legacy feature! Old 'def' command -- use 'define' instead ### Legacy feature! Old 'def' command -- use 'define' instead ### Introduced fixed type variable(s): 'a in "P__" or "Q__" ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Introduced fixed type variable(s): 'a in "xs__" class preorder = ord + assumes "less_le_not_le": "\x y. (x < y) = (x \ y \ \ y \ x)" and "order_refl": "\x. x \ x" and "order_trans": "\x y z. \x \ y; y \ z\ \ x \ z" class monoid_add = semigroup_add + zero + assumes "add_0_left": "\a. (0::'a) + a = a" and "add_0_right": "\a. a + (0::'a) = a" ### theory "Coinductive.Coinductive_List" ### 7.419s elapsed time, 14.120s cpu time, 1.132s GC time Loading theory "Coinductive.Coinductive_List_Prefix" (required by "Coinductive.Coinductive") Testing conjecture with Quickcheck-random... instantiation llist :: (type) order less_eq_llist == less_eq :: 'a llist \ 'a llist \ bool less_llist == less :: 'a llist \ 'a llist \ bool Quickcheck found a counterexample: xs = LCons a\<^sub>1 (LCons a\<^sub>1 LNil) Loading theory "Coinductive.Hamming_Stream" (required by "Coinductive.Coinductive_Examples") instantiation llist :: (type) order_bot bot_llist == bot :: 'a llist instantiation llist :: (type) semilattice_inf inf_llist == inf :: 'a llist \ 'a llist \ 'a llist instantiation llist :: (type) ccpo Sup_llist == Sup :: 'a llist set \ 'a llist ### theory "Coinductive.Coinductive_List_Prefix" ### 0.576s elapsed time, 1.024s cpu time, 0.000s GC time Loading theory "Coinductive.Koenigslemma" (required by "Coinductive.Coinductive_Examples") Proofs for coinductive predicate(s) "pathsp" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the coinduction rule ... Proving the simplification rules ... Proofs for inductive predicate(s) "reachable_viap" Proving monotonicity ... Proving the introduction rules ... Proving the elimination rules ... Proving the induction rule ... Proving the simplification rules ... ### theory "Coinductive.Koenigslemma" ### 0.374s elapsed time, 0.664s cpu time, 0.000s GC time Loading theory "Coinductive.LMirror" (required by "Coinductive.Coinductive_Examples") class ord = type + fixes less_eq :: "'a \ 'a \ bool" and less :: "'a \ 'a \ bool" consts lmirror_aux :: "'a llist \ 'a llist \ 'a llist" ### Ambiguous input (line 28 of "~~/afp/thys/Coinductive/Examples/Hamming_Stream.thy") produces 2 parse trees: ### ("\<^const>HOL.Trueprop" ### ("\<^const>HOL.eq" ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case2" ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case1" ("_position" LNil) ("_position" LNil)))) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ### ("_applC" ("_position" lhd) ("_position" xs)) ### ("_applC" ("_position" lhd) ("_position" ys))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs') ("_position" ys))))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ### ("_applC" ("_position" lhd) ("_position" ys)) ### ("_applC" ("_position" lhd) ("_position" xs))) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs) ("_position" ys'))) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs') ### ("_position" ys'))))))))))))) ### ("\<^const>HOL.Trueprop" ### ("\<^const>HOL.eq" ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ### ("_applC" ("_position" lhd) ("_position" xs)) ### ("_applC" ("_position" lhd) ("_position" ys))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs') ("_position" ys))))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ### ("_applC" ("_position" lhd) ("_position" ys)) ### ("_applC" ("_position" lhd) ("_position" xs))) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs) ("_position" ys'))) ### ("_applC" ("_position" lmerge) ### ("_cargs" ("_position" xs') ### ("_position" ys'))))))))))))))) ### Fortunately, only one parse tree is well-formed and type-correct, ### but you may still want to disambiguate your grammar or your input. ### Ignoring duplicate rewrite rule: ### lnull (lmirror_aux ?acc1 ?xs1) \ lnull ?xs1 \ lnull ?acc1 consts lmerge :: "'a llist \ 'a llist \ 'a llist" ### theory "Coinductive.LMirror" ### 0.237s elapsed time, 0.420s cpu time, 0.000s GC time Loading theory "Coinductive.Lazy_LList" (required by "Coinductive.Lazy_TLList") ### Ignoring duplicate rewrite rule: ### lnull (lmerge ?xs1 ?ys1) \ lnull ?xs1 \ lnull ?ys1 ### Ambiguous input (line 85 of "~~/afp/thys/Coinductive/Examples/Hamming_Stream.thy") produces 2 parse trees: ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" lmerge) ### ("_pattern" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ("_position" x) ### ("_position" y)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs') ("_position" ys)))))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ("_position" y) ### ("_position" x)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs) ### ("_position" ys')))))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs') ### ("_position" ys')))))))))))))))) ### ("\<^const>Pure.eq" ("_position" F) ### ("_lambda" ### ("_pttrns" ("_position" lmerge) ### ("_pattern" ("_position" xs) ("_position" ys))) ### ("_case_syntax" ("_position" xs) ### ("_case2" ("_case1" ("_position" LNil) ("_position" LNil)) ### ("_case2" ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ("_position" xs'))) ### ("_case_syntax" ("_position" ys) ### ("_case1" ("_position" LNil) ("_position" LNil)))) ### ("_case1" ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ("_position" ys'))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ("_position" x) ### ("_position" y)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" x) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs') ("_position" ys)))))) ### ("\<^const>HOL.If" ### ("\<^const>Orderings.ord_class.less" ("_position" y) ### ("_position" x)) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs) ("_position" ys')))))) ### ("_applC" ("_position" LCons) ### ("_cargs" ("_position" y) ### ("_applC" ("_position" curry) ### ("_cargs" ("_position" lmerge) ### ("_cargs" ("_position" xs') ### ("_position" ys')))))))))))))) ### Fortunately, only one parse tree is well-formed and type-correct, ### but you may still want to disambiguate your grammar or your input. class linorder = order + assumes "linear": "\x y. x \ y \ y \ x" ### theory "Coinductive.Lazy_LList" ### 0.776s elapsed time, 1.108s cpu time, 0.272s GC time Loading theory "Coinductive.Quotient_Coinductive_List" (required by "Coinductive.Coinductive") ### theory "Coinductive.Hamming_Stream" ### 1.695s elapsed time, 2.700s cpu time, 0.272s GC time Loading theory "Coinductive.TLList" (required by "Coinductive.Coinductive") ### theory "Coinductive.Quotient_Coinductive_List" ### 0.920s elapsed time, 1.544s cpu time, 0.000s GC time Loading theory "Coinductive.Coinductive_Stream" (required by "Coinductive.Coinductive") overloading terminal0 \ terminal0 :: ('a, 'b) tllist \ 'b consts unfold_tllist :: "('a \ bool) \ ('a \ 'b) \ ('a \ 'c) \ ('a \ 'a) \ 'a \ ('c, 'b) tllist" consts unfold_stream :: "('a \ 'b) \ ('a \ 'a) \ 'a \ 'b stream" consts tllist_of_llist :: "'a llist \ ('a, 'b) tllist" consts llist_of_tllist :: "('a, 'b) tllist \ 'a llist" locale stream_from_llist_setup ### theory "Coinductive.Coinductive_Stream" ### 1.294s elapsed time, 2.260s cpu time, 0.000s GC time Loading theory "Coinductive.LList_CCPO_Topology" (required by "Coinductive.Coinductive_Examples") instantiation llist :: (type) ccpo_topology open_llist == open :: 'a llist set \ bool consts edrop :: "enat \ 'a list \ 'a list" ### theory "Coinductive.TLList" ### 3.754s elapsed time, 6.152s cpu time, 0.704s GC time Loading theory "Coinductive.Lazy_TLList" consts up :: "'a \ 'a list \ 'a list" ### theory "Coinductive.Lazy_TLList" ### 0.598s elapsed time, 0.976s cpu time, 0.000s GC time Loading theory "Coinductive.Quotient_TLList" (required by "Coinductive.Coinductive") Found termination order: "case_sum (\p. size_list (nat \ abs) (snd p)) (\p. size_list (nat \ abs) (snd p)) <*mlex*> {}" ### theory "Coinductive.LList_CCPO_Topology" ### 2.716s elapsed time, 4.292s cpu time, 0.704s GC time Loading theory "Coinductive.TLList_CCPO" (required by "Coinductive.Coinductive_Examples" via "Coinductive.TLList_CCPO_Examples") locale tllist_pf fixes b :: "'b" ### theory "Coinductive.TLList_CCPO" ### 0.819s elapsed time, 1.624s cpu time, 0.000s GC time Loading theory "Coinductive.TLList_CCPO_Examples" (required by "Coinductive.Coinductive_Examples") ### theory "Coinductive.Quotient_TLList" ### 1.289s elapsed time, 2.444s cpu time, 0.000s GC time Loading theory "Coinductive.Coinductive" ### Ignoring duplicate rewrite rule: ### \mcont ?luba1 ?orda1 Sup op \ ?f1; ### mcont ?luba1 ?orda1 Sup op \ ?g1\ ### \ ccpo.admissible ?luba1 ?orda1 ### (\x. ?f1 x \ ?g1 x) \ ### True ### theory "Coinductive.TLList_CCPO_Examples" ### 0.169s elapsed time, 0.336s cpu time, 0.000s GC time Loading theory "Coinductive.Coinductive_Examples" ### theory "Coinductive.Coinductive" ### 1.376s elapsed time, 2.500s cpu time, 0.364s GC time Testing conjecture with Quickcheck-exhaustive... Quickcheck found a counterexample: xs = LCons a\<^sub>1 LNil Evaluated terms: LNil = LNil Testing conjecture with Quickcheck-narrowing... ### theory "Coinductive.Coinductive_Examples" ### 2.353s elapsed time, 4.116s cpu time, 0.364s GC time [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4285832/isabelle_quickcheck_narrowing ... ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a ### Ignoring duplicate rewrite rule: ### \x\?A1. \ lnull x \ ### lhd (lSup ?A1) \ ### THE x. x \ lhd ` (?A1 \ {xs. \ lnull xs}) ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4287986/isabelle_quickcheck_narrowing ... ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4288070/isabelle_quickcheck_narrowing ... Quickcheck found no counterexample. ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Ignoring duplicate rewrite rule: ### class.ccpo lSup op \ (mk_less op \) \ True ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Introduced fixed type variable(s): 'b in "zs__" ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Legacy feature! Old 'def' command -- use 'define' instead ### Metis: Unused theorems: "Coinductive_List.lappend_llist_of_llist_of" ### Metis: Unused theorems: "Coinductive_List.lfinite_lappend", "Coinductive_List.lfinite_llist_of", "Coinductive_List.list_of_lappend", "Coinductive_List.list_of_llist_of" ### Legacy feature! Old 'def' command -- use 'define' instead ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Introduced fixed type variable(s): 'b in "xs__" ### Metis: Unused theorems: "Coinductive_Nat.enat_le_plus_same_2" ### Metis: Unused theorems: "Coinductive_Nat.enat_le_plus_same_1" ### Legacy feature! Old 'def' command -- use 'define' instead ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x ### Legacy feature! Old 'def' command -- use 'define' instead ### Legacy feature! Old 'def' command -- use 'define' instead ### Legacy feature! Old 'def' command -- use 'define' instead ### Rule already declared as introduction (intro) ### ?P ?x \ \x. ?P x val zeros = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val lhd = 0: int val ltl = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val ltl' = SOME (1, Lazy_llist fn): (int * int Isabelle4316274.Generated_Code.llist) option val ltake = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val ldrop = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val list_of = [0, 1]: int list val ltakeWhile = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val ldropWhile = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist val hd = 0: int val lfilter = Lazy_llist fn: int Isabelle4316274.Generated_Code.llist Testing conjecture with Quickcheck-random... Quickcheck found a counterexample: xs = TCons a\<^sub>1 (TCons a\<^sub>1 (TNil a\<^sub>1)) x = a\<^sub>1 Testing conjecture with Quickcheck-narrowing... Testing conjecture with Quickcheck-exhaustive... Quickcheck found a counterexample: xs = TCons a\<^sub>1 (TNil a\<^sub>1) x = a\<^sub>1 Evaluated terms: TNil x = TNil a\<^sub>1 ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### \?r ?a ?b; ?s ?b ?c\ \ (?r OO ?s) ?a ?c ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### \?r ?a ?b; ?s ?b ?c\ \ (?r OO ?s) ?a ?c ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### \?r ?a ?b; ?s ?b ?c\ \ (?r OO ?s) ?a ?c ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### \?r ?a ?b; ?s ?b ?c\ \ (?r OO ?s) ?a ?c ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### \?r ?a ?b; ?s ?b ?c\ \ (?r OO ?s) ?a ?c [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4321004/isabelle_quickcheck_narrowing ... [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4322970/isabelle_quickcheck_narrowing ... [1 of 4] Compiling Typerep ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Typerep.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Typerep.o ) [2 of 4] Compiling Generated_Code ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Generated_Code.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Generated_Code.o ) [3 of 4] Compiling Narrowing_Engine ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Narrowing_Engine.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Narrowing_Engine.o ) [4 of 4] Compiling Main ( /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Main.hs, /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/Main.o ) Linking /tmp/isabelle-jenkins/process3597726338088514653/Quickcheck_Narrowing4324734/isabelle_quickcheck_narrowing ... Quickcheck found no counterexample. *** exception THM 0 raised (line 328 of "drule.ML"): *** OF: no unifiers *** \closed ?s; \x. isCont ?f x\ *** \ closed (?f -` ?s) *** isCont (\x. (f x, g x)) ?a *** closed {(x, y). llist_all2 ?R x y} *** At command "using" (line 194 of "~~/afp/thys/Coinductive/Examples/LList_CCPO_Topology.thy") ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Ignoring duplicate rewrite rule: ### ((\x. x) \ ?a1) (at ?a1 within ?s1) \ ### True ### Rule already declared as introduction (intro) ### (\x y. ?A x y \ ?B (?f x) (?g y)) \ ### (?A ===> ?B) ?f ?g ### Rule already declared as introduction (intro) ### ((\x. x) \ ?a) (at ?a within ?s) ### Rule already declared as introduction (intro) ### ((\x. ?k) \ ?k) ?F ### Rule already declared as introduction (intro) ### (?f \ ?x) ?F \ ### ((\x. ereal (?f x)) \ ereal ?x) ?F ### Rule already declared as introduction (intro) ### (?f \ ?x) ?F \ ### ((\x. - ?f x) \ - ?x) ?F ### Rule already declared as introduction (intro) ### \\?c\ \ \; ### (?f \ ?x) ?F\ ### \ ((\x. ?c * ?f x) \ ?c * ?x) ?F ### Rule already declared as introduction (intro) ### \?x \ 0; (?f \ ?x) ?F\ ### \ ((\x. ?c * ?f x) \ ?c * ?x) ?F ### Rule already declared as introduction (intro) ### \?y \ - \; ?x \ - \; ### (?f \ ?x) ?F\ ### \ ((\x. ?f x + ?y) \ ?x + ?y) ?F ### Rule already declared as introduction (intro) ### \\?y\ \ \; ### (?f \ ?x) ?F\ ### \ ((\x. ?f x + ?y) \ ?x + ?y) ?F val zeros = Lazy_tllist fn: (int, int) Isabelle4334060.Generated_Code.tllist val thd = 0: int val ttl = Lazy_tllist fn: (int, int) Isabelle4334060.Generated_Code.tllist val ttl' = Inl (0, Lazy_tllist fn): (int * (int, int) Isabelle4334060.Generated_Code.tllist, int) Isabelle4334060.Generated_Code.sum val tdropn = Lazy_tllist fn: (int, int) Isabelle4334060.Generated_Code.tllist val tfilter = Lazy_tllist fn: (int, int) Isabelle4334060.Generated_Code.tllist ### Rule already declared as introduction (intro) ### (\x. ?f x = ?g x) \ ?f = ?g ### Rule already declared as introduction (intro) ### \?P ?a; \x. ?P x \ x = ?a\ ### \ (THE x. ?P x) = ?a ### Rule already declared as introduction (intro) ### (\x. ?f x = ?g x) \ ?f = ?g ### Rule already declared as introduction (intro) ### (\x. ?f x = ?g x) \ ?f = ?g ### Ignoring duplicate introduction (intro) ### (\x. ?f x = ?g x) \ ?f = ?g ### Metis: Unused theorems: "??.unknown" ### Metis: Unused theorems: "??.unknown" ### Ignoring duplicate rewrite rule: ### tllist_all2 op = op = \ op = isabelle document -o 'pdf' -n 'document' -t '' /media/data/jenkins/workspace/afp-repo-afp/browser_info/AFP/Coinductive/document 2>&1 isabelle document -o 'pdf' -n 'outline' -t '/proof,/ML' /media/data/jenkins/workspace/afp-repo-afp/browser_info/AFP/Coinductive/outline 2>&1 This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty Including comment 'isadelimproof' Excluding comment 'isatagproof' Including comment 'isadelimML' Excluding comment 'isatagML') (./isabellesym.sty ) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) No file root.aux. (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) [1{/var/lib/texmf/font s/map/pdftex/updmap/pdftex.map}] (./session.tex (./Coinductive_Nat.tex [2] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [3] [4] Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [5] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [6] [7] [8] [9] [10] [11]) (./Coinductive_List.tex [12] [13] [14] [15] [16] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [17] [18] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [19] [20] [21] [22] [23] [24] [25] [26] [27] [28] [29] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [30] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [31] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. [32] [33] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [34] [35] [36] [37] [38] [39] [40] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [41] [42] [43] [44] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [45] [46] [47] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [48] [49] [50] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [51] [52] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset [53] [54] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [55] [56] [57] [58] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [59] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [60] [61] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [62] [63] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [64] [65] [66] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [67] [68] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [69] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [70] [71] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [72] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [73] [74] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [75] [76] [77] [78] [79]) (./Coinductive_List_Prefix.tex [80] [81]) (./Coinductive_Stream.tex [82] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. [83] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [84] [85] [86] [87] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [88] [89] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. [90]) (./TLList.tex [91] [92] [93] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [94] [95] [96] [97] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. [98] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. [99] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [100] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. [101] Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [102] [103] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [104] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [105] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [106] [107] [108]) (./Quotient_Coinductive_List.tex [109] [110] [111]) (./Quotient_TLList.tex Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [112] [113] Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [114] Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] ) (./Coinductive.tex) (./Lazy_LList.tex [115] Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [116] [117] [118] [119] [120] [121]) (./Lazy_TLList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [122] [123] [124] [125]) (./CCPO_Topology.tex [126] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [127] [128] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. ) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [129] [130] [131] [132] [133] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [134] [135]) (./TLList_CCPO_Examples.tex [136]) (./Koenigslemma.tex Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [137]) (./LMirror.tex [138] [139] [140]) (./Hamming_Stream.tex [141] [142] Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] [143] [144] [145]) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case [146] Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ [147] Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] [148] Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption [149] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [150] Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [151] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion ) (./Coinductive_Examples.tex [152])) [153] (./root.aux) Package rerunfilecheck Warning: File `root.out' has changed. (rerunfilecheck) Rerun to get outlines right (rerunfilecheck) or use package `bookmark'. ) (see the transcript file for additional information) Output written on root.pdf (153 pages, 449204 bytes). Transcript written on root.log. This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty Including comment 'isadelimproof' Excluding comment 'isatagproof' Including comment 'isadelimML' Excluding comment 'isatagML') (./isabellesym.sty ) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) (./root.aux) (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (./root.out) (./root.out) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) (./root.toc [1{/var/li b/texmf/fonts/map/pdftex/updmap/pdftex.map}] [2] [3]) [4] (./session.tex (./Coinductive_Nat.tex [5] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [6] [7] Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [8] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [9] [10] [11] [12] [13] [14]) (./Coinductive_List.tex [15] [16] [17] [18] [19] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [20] [21] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [22] [23] [24] [25] [26] [27] [28] [29] [30] [31] [32] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [33] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [34] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. [35] [36] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [37] [38] [39] [40] [41] [42] [43] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [44] [45] [46] [47] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [48] [49] [50] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [51] [52] [53] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [54] [55] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset [56] [57] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [58] [59] [60] [61] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [62] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [63] [64] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [65] [66] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [67] [68] [69] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [70] [71] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [72] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [73] [74] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [75] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [76] [77] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [78] [79] [80] [81] [82]) (./Coinductive_List_Prefix.tex [83] [84]) (./Coinductive_Stream.tex [85] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. [86] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [87] [88] [89] [90] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [91] [92] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. [93]) (./TLList.tex [94] [95] [96] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [97] [98] [99] [100] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. [101] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. [102] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [103] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. [104] Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [105] [106] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [107] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [108] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [109] [110] [111]) (./Quotient_Coinductive_List.tex [112] [113] [114]) (./Quotient_TLList.tex Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [115] [116] Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [117] Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] ) (./Coinductive.tex) (./Lazy_LList.tex [118] Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [119] [120] [121] [122] [123] [124]) (./Lazy_TLList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [125] [126] [127] [128]) (./CCPO_Topology.tex [129] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [130] [131] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. ) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [132] [133] [134] [135] [136] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [137] [138]) (./TLList_CCPO_Examples.tex [139]) (./Koenigslemma.tex Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [140]) (./LMirror.tex [141] [142] [143]) (./Hamming_Stream.tex [144] [145] Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] [146] [147] [148]) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case [149] Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ [150] Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] [151] Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption [152] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [153] Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [154] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion ) (./Coinductive_Examples.tex [155])) [156] (./root.aux) ) (see the transcript file for additional information) Output written on root.pdf (156 pages, 468676 bytes). Transcript written on root.log. This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty Including comment 'isadelimproof' Excluding comment 'isatagproof' Including comment 'isadelimML' Excluding comment 'isatagML') (./isabellesym.sty ) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) (./root.aux) (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (./root.out) (./root.out) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) (./root.toc [1{/var/li b/texmf/fonts/map/pdftex/updmap/pdftex.map}] [2] [3]) [4] (./session.tex (./Coinductive_Nat.tex [5] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [6] [7] Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [8] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [9] [10] [11] [12] [13] [14]) (./Coinductive_List.tex [15] [16] [17] [18] [19] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [20] [21] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [22] [23] [24] [25] [26] [27] [28] [29] [30] [31] [32] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [33] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [34] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. [35] [36] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [37] [38] [39] [40] [41] [42] [43] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [44] [45] [46] [47] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [48] [49] [50] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [51] [52] [53] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [54] [55] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset [56] [57] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [58] [59] [60] [61] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [62] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [63] [64] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [65] [66] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [67] [68] [69] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [70] [71] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [72] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [73] [74] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [75] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [76] [77] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [78] [79] [80] [81] [82]) (./Coinductive_List_Prefix.tex [83] [84]) (./Coinductive_Stream.tex [85] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. [86] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [87] [88] [89] [90] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [91] [92] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. [93]) (./TLList.tex [94] [95] [96] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [97] [98] [99] [100] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. [101] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. [102] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [103] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. [104] Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [105] [106] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [107] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [108] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [109] [110] [111]) (./Quotient_Coinductive_List.tex [112] [113] [114]) (./Quotient_TLList.tex Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [115] [116] Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [117] Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] ) (./Coinductive.tex) (./Lazy_LList.tex [118] Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [119] [120] [121] [122] [123] [124]) (./Lazy_TLList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [125] [126] [127] [128]) (./CCPO_Topology.tex [129] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [130] [131] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. ) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [132] [133] [134] [135] [136] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [137] [138]) (./TLList_CCPO_Examples.tex [139]) (./Koenigslemma.tex Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [140]) (./LMirror.tex [141] [142] [143]) (./Hamming_Stream.tex [144] [145] Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] [146] [147] [148]) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case [149] Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ [150] Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] [151] Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption [152] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [153] Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [154] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion ) (./Coinductive_Examples.tex [155])) [156] (./root.aux) ) (see the transcript file for additional information) Output written on root.pdf (156 pages, 468680 bytes). Transcript written on root.log. This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty) (./isabellesym.sty) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) No file root.aux. (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) [1{/var/lib/texmf/font s/map/pdftex/updmap/pdftex.map}] (./session.tex (./Coinductive_Nat.tex [2] [3] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [4] Overfull \hbox (25.18492pt too wide) in paragraph at lines 655--668 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus one[]enat[]def zero[]enat[]def eSuc[]def epred[]numeral[]def Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [5] Overfull \hbox (59.08212pt too wide) in paragraph at lines 735--748 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]coexhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/ 10 case[]product enat[]coexhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 simp[ ]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus$\OT1/cmr/m/n/10 )$[] Overfull \hbox (26.72835pt too wide) in paragraph at lines 771--784 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 )$[] [6] Overfull \hbox (23.20164pt too wide) in paragraph at lines 952--969 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 bot[]enat[]def Sup[]enat[]def epred[]Max inj[ ]on[]def neq[]zero[]conv[]eSuc [7] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [8] [9] Overfull \hbox (64.72255pt too wide) in paragraph at lines 1437--1450 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y m rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all$\OML/cmm/m/it/10 ;$ [10] Overfull \hbox (22.26717pt too wide) in paragraph at lines 1545--1558 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m x y rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (22.99493pt too wide) in paragraph at lines 1563--1576 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m k rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (53.3571pt too wide) in paragraph at lines 1625--1627 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Sup[]enat[]def Max[]enat[]minus1 finite[]less Than[]enat[]iff enat[]diff[]cancel[]left [11] [12] Overfull \hbox (11.05505pt too wide) in paragraph at lines 1990--2003 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]eadd1 mcont[]eadd2 [13] Overfull \hbox (6.50609pt too wide) in paragraph at lines 2143--2145 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule finite[ ]imageD$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 inj[]onI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 max[]de f split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [14] Overfull \hbox (52.5326pt too wide) in paragraph at lines 2239--2252 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]max[]enat1 mcont[]max[]enat2 [15] [16]) (./Coinductive_List.tex [17] [18] [19] [20] [21] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. [22] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [23] [24] [25] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [26] [27] Overfull \hbox (16.47273pt too wide) in paragraph at lines 1960--1962 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys zs$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv LCons[]lprefix[]conv$\OML/cmm/m/it/10 ;$ [28] Overfull \hbox (1.58864pt too wide) in paragraph at lines 2103--2116 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSup$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 lprefix[]lhdD in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]e quality$\OT1/cmr/m/n/10 )$[] [29] Overfull \hbox (24.56723pt too wide) in paragraph at lines 2175--2188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 expand$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto si mp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image lhd[]lSup exI LCons[]im age[]Int[]not[]lnull Overfull \hbox (14.04483pt too wide) in paragraph at lines 2290--2293 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 ?LCons \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/i t/10 the[]equality dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lprefix[]lhdD in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]image[]eqI$\OT1/cmr/m/n/10 )$[] [30] [31] [32] [33] Overfull \hbox (0.19804pt too wide) in paragraph at lines 2834--2847 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF lnil$\OT1/cmr/m/n/ 10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (24.52327pt too wide) in paragraph at lines 2874--2887 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 monotone[]if[]bot$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 f$\OT1/cmr/m/n/10 =$$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it /10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 f $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 lhd xs$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 ltl xs$\OT1/cmr/m/n/10 )$ \OT1 /cmr/m/it/10 xs \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 bound$\OT1/cmr/m/n/10 =$\ OT1/cmr/m/it/10 LNil$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto Overfull \hbox (2.5006pt too wide) in paragraph at lines 2874--2887 \OT1/cmr/m/it/10 4 3 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 split simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv LCons[]lprefix[]conv dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mo no-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.96495pt too wide) in paragraph at lines 2915--2919 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 ob-tain \OT1/cm r/m/it/10 x xs \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 LCons x xs $\OMS/cmsy/m/ n/10 2$ \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv$\OT1 /cmr/m/n/10 )$[] Overfull \hbox (3.45793pt too wide) in paragraph at lines 2922--2924 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force dest$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF cha in$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 LCons[]lprefix[]conv lprefix[]LCons[]conv [34] Overfull \hbox (11.3537pt too wide) in paragraph at lines 3014--3036 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term llist$\OML/c mm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @ $$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 fixp[]rule[]uc$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$ \OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]strong[]in duct[]uc$\OMS/cmsy/m/n/10 g$ Overfull \hbox (10.92476pt too wide) in paragraph at lines 3050--3058 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [35] Overfull \hbox (10.92476pt too wide) in paragraph at lines 3225--3233 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [36] Overfull \hbox (11.56499pt too wide) in paragraph at lines 3404--3406 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSu p$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 dest$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ] $ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]equality$ \OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ [37] [38] [39] [40] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [41] Overfull \hbox (16.78535pt too wide) in paragraph at lines 3905--3907 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs$ [] $ rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]induct$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Nil lappend[]llis t[]of[]llist[]of$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ] $ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [42] [43] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Overfull \hbox (15.20331pt too wide) in paragraph at lines 4386--4399 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 epred[]iadd1 [44] [45] Overfull \hbox (10.92476pt too wide) in paragraph at lines 4665--4673 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (18.88669pt too wide) in paragraph at lines 4677--4679 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 subst $\OT1/cmr/m /n/10 ($\OT1/cmr/m/it/10 1 2 3$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lfp$\OML/cmm /m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (17.23381pt too wide) in paragraph at lines 4692--4705 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/ 10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Overfull \hbox (19.53375pt too wide) in paragraph at lines 4711--4728 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it /10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [46] Overfull \hbox (17.11995pt too wide) in paragraph at lines 4940--4953 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\ OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff [47] [48] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5331--5339 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [49] [50] [51] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5786--5794 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [52] [53] [54] [55] Overfull \hbox (25.67209pt too wide) in paragraph at lines 6689--6693 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 LCons \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/1 0 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 )$$($\OT1/cm r/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]Suc[]right$\O T1/cmr/m/n/10 )$[] [56] Overfull \hbox (68.23685pt too wide) in paragraph at lines 6786--6790 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Cons \OT1/cmr/bx/n/10 thus \OT1/cm r/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (27.84201pt too wide) in paragraph at lines 6882--6895 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldrop[]LCons iadd[]Suc[]righ t split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it /10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.39761pt too wide) in paragraph at lines 6900--6917 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltake[]LCons ldrop[]LCons sp lit$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [57] [58] [59] Overfull \hbox (1.621pt too wide) in paragraph at lines 7327--7330 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ex I$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 = $\OT1/cmr/m/it/10 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/1 0 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (19.0108pt too wide) in paragraph at lines 7336--7338 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 wh ere \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc n \OT1/cmr/bx/n/1 0 for \OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ileI1 simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] [60] Overfull \hbox (28.40157pt too wide) in paragraph at lines 7638--7651 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis eSuc[]enat eSu c[]plus[]1 ltake[]plus[]conv[]lappend ldrop[]enat ldropn[]Suc[]conv[]ldropn [61] [62] [63] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [64] Overfull \hbox (5.19078pt too wide) in paragraph at lines 8236--8249 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def lnull[]d ef neq[]LNil[]conv [65] [66] Overfull \hbox (4.94086pt too wide) in paragraph at lines 8503--8516 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 prefix[]def lprefix[]conv[]lappend$\OT1/cmr/m/n/1 0 )$$($\OT1/cmr/m/it/10 metis lfinite[]lappend lfinite[]llist[]of Overfull \hbox (21.38031pt too wide) in paragraph at lines 8611--8616 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lSup A$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 enat n \OT1/c mr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 lfinite[]conv[]llength[]enat Overfull \hbox (2.40771pt too wide) in paragraph at lines 8620--8623 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 fi-nite $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 llength ` A$\OT1/cmr/m/n/10 )$ \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ( $\OT1/cmr/m/it/10 rule finite[]subset$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 sim p add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 finite[]lessThan[]enat[]iff$\OT1/cmr/ m/n/10 )$[] [67] Overfull \hbox (13.92545pt too wide) in paragraph at lines 8799--8812 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llcp[]eq[]0[]iff epred[]llcp [68] Overfull \hbox (10.21999pt too wide) in paragraph at lines 8818--8831 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 llcp[]eq[]0[]iff Overfull \hbox (14.39069pt too wide) in paragraph at lines 8836--8849 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis add[]0[]right lappend[]LNil2 llcp[]LNil1 llcp[]lappend[]same lprefix[]conv[]lappend$\OT1/cmr /m/n/10 )$[] Overfull \hbox (52.74213pt too wide) in paragraph at lines 8897--8899 \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/ cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 iadd[]Suc[]right zero []enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[ ] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [69] Overfull \hbox (5.10889pt too wide) in paragraph at lines 9073--9086 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff Overfull \hbox (14.78528pt too wide) in paragraph at lines 9140--9148 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [70] Overfull \hbox (2.44716pt too wide) in paragraph at lines 9295--9298 [][] \OT1/cmr/bx/n/10 thus \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr /m/n/10 ($\OT1/cmr/m/it/10 cases ys n rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 case[]product co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/1 0 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr/m/it/10 simp[]all[] [71] [72] [73] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9748--9761 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9767--9780 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9788--9805 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [74] Overfull \hbox (10.92476pt too wide) in paragraph at lines 9859--9867 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (0.88739pt too wide) in paragraph at lines 9893--9906 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr /m/it/10 simp[] Overfull \hbox (3.18733pt too wide) in paragraph at lines 9912--9925 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cm r/m/it/10 simp[] [75] [76] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset Overfull \hbox (23.46579pt too wide) in paragraph at lines 10431--10444 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv [77] [78] Overfull \hbox (4.60457pt too wide) in paragraph at lines 10598--10606 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 llength[]ltakeWhile[]all$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 llen gth[]eq[]infty[]conv[]lfinite$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1 /cmr/m/n/10 ]$[] Overfull \hbox (34.96571pt too wide) in paragraph at lines 10694--10707 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n /10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [79] Overfull \hbox (6.35873pt too wide) in paragraph at lines 10905--10918 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]eq[]infty[]conv[]l finite lfinite[]ltakeWhile$\OT1/cmr/m/n/10 )$[] Overfull \hbox (43.52377pt too wide) in paragraph at lines 10925--10938 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]ldrop llength[]lta keWhile[]all ltakeWhile[]all[]conv [80] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [81] Overfull \hbox (31.74066pt too wide) in paragraph at lines 11315--11317 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 step llist[]all2[]llengthD [82] Overfull \hbox (25.92279pt too wide) in paragraph at lines 11331--11333 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases lnull xs $\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 step simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cm r/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lnth[ ]0[]conv[]lhd$\OT1/cmr/m/n/10 )$[] [83] Overfull \hbox (37.6261pt too wide) in paragraph at lines 11639--11644 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth ys n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 ltake $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llength xs$\OT 1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 n \OT1/ cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lnth[]ltake$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (4.15424pt too wide) in paragraph at lines 11644--11649 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lappend xs xs$ [] $$\OT1 /cmr/m/n/10 )$ \OT1/cmr/m/it/10 n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth xs n \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 lnth[]lappend1$\OT1/cmr/m/n/10 )$[] [84] Overfull \hbox (15.4463pt too wide) in paragraph at lines 11688--11690 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 neq[]LNil[]conv lnul l[]def LNil[]eq[]lmap Overfull \hbox (24.38661pt too wide) in paragraph at lines 11696--11698 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lnullD llis t[]all2[]lhdD llist[]all2[]ltlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (7.40894pt too wide) in paragraph at lines 11742--11749 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [85] Overfull \hbox (12.14566pt too wide) in paragraph at lines 11911--11913 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image dest$\OT1/cmr/m/n/10 :$ \ OT1/cmr/m/it/10 Y llist[]all2[]lnullD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 rev[]image[]eqI$\OT1/cmr/m/n/10 )$$+$[] [86] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. [87] Overfull \hbox (18.37143pt too wide) in paragraph at lines 12252--12256 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Suc \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x s$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$ \OT1/cmr/m/it/10 llast[]LCons$\OT1/cmr/m/n/10 )$[] [88] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [89] Overfull \hbox (5.61943pt too wide) in paragraph at lines 12468--12472 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chain[]lprefix[]ltl chain in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldistinct[]ltlI Overfull \hbox (17.75882pt too wide) in paragraph at lines 12506--12508 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ldistinct[]lSup chain[]imageI mcont[ ]monoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [90] [91] Overfull \hbox (0.21182pt too wide) in paragraph at lines 12872--12889 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv des t$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lset[]lzipD2$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [92] Overfull \hbox (3.13603pt too wide) in paragraph at lines 13020--13025 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 us -ing \OT1/cmr/m/it/10 chain sorted \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]ltl lsorted[]ltlI$\OT1/cmr/m/n/10 )$[] [93] Overfull \hbox (11.49773pt too wide) in paragraph at lines 13106--13108 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lsorted[]lSup chain[]imageI mcont[]m onoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (12.42061pt too wide) in paragraph at lines 13121--13134 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 admissibleI$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 aut o dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lsorted[]lprefixD$\OT1/cmr/m/n/10 [$ \OT1/cmr/m/it/10 rotated$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]lSup$\OT1/cmr/m/n/10 )$[] Overfull \hbox (4.57834pt too wide) in paragraph at lines 13157--13170 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct n ar-bi-trary $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 f astforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldropn[]Suc lsorted[]LCon s$ [] $ ldropn[]lnull [94] Overfull \hbox (1.39157pt too wide) in paragraph at lines 13303--13310 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lsorted[]coinduct$ [] $$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mon o-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [95] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [96] [97] [98] [99] [100] [101] [102] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [103] Overfull \hbox (5.09007pt too wide) in paragraph at lines 14626--14639 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 drule eq[]LConsD$\OT 1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m /it/10 exI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltl[]lfilter o[]def ldr opWhile[]eq[]LNil[]iff [104] [105] [106] [107] Overfull \hbox (14.26587pt too wide) in paragraph at lines 15252--15254 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]snocL1[]conv[]LCons2$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 symmetric$\OML/cmm/m/it/10 ;$ \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 lappend [108] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [109] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [110] [111] [112] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [113] [114] Overfull \hbox (13.61642pt too wide) in paragraph at lines 16286--16290 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 concat[]xss$ [] $ nth[]n \OT 1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 xss \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lnth[]lappe nd2 lappend[]lnull1$\OT1/cmr/m/n/10 )$[] [115] Overfull \hbox (1.33876pt too wide) in paragraph at lines 16330--16332 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/ cmr/m/n/10 ($\OT1/cmr/m/it/10 1 2$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 atLeast0L essThan$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$$($\O T1/cmr/m/it/10 subst sum[]add[]nat[]ivl$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 si mp[]all$\OT1/cmr/m/n/10 )$[] [116] [117] Overfull \hbox (4.77174pt too wide) in paragraph at lines 16574--16576 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 lfilter[]eq[]LConsD$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF []LCons x xs $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lfi l-ter $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 xs$\OML/cmm/m/i t/10 :$ $\OMS/cmsy/m/n/10 :$ \OT1/cmr/m/it/10 lnull xs$\OT1/cmr/m/n/10 )$ \OT1/ cmr/m/it/10 xss[]$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$]$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [118] [119] [120] [121] [122] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [123] [124] [125] [126] Overfull \hbox (11.00165pt too wide) in paragraph at lines 18136--18149 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set1[]pre[]llist[]def rel[]set[]def Overfull \hbox (11.00165pt too wide) in paragraph at lines 18155--18168 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set2[]pre[]llist[]def rel[]set[]def [127] [128] [129]) (./Coinductive_List_Prefix.tex [130] [131] Overfull \hbox (17.24495pt too wide) in paragraph at lines 330--336 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 Sup[]llist[]def less[]eq[]llist[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 abs[]def$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]upper llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]least$\OT1/cmr/m/n/10 )$[] ) (./Coinductive_Stream.tex [132] [133] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [134] [135] [136] [137] Overfull \hbox (1.53853pt too wide) in paragraph at lines 1044--1057 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]stream[]def cr[]stream[]def in-tro$\OT1/ cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 rel[]funI rel-comppI rel[]setI [138] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. [139] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [140] Overfull \hbox (6.55463pt too wide) in paragraph at lines 1618--1624 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 bot[]enat[]def in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 admiss ible[]all admissible[]imp admissible[]eq[]mcontI Overfull \hbox (32.81557pt too wide) in paragraph at lines 1702--1707 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 step \OT1/cmr/bx/n/10 un-fol d-ing \OT1/cmr/m/it/10 eq \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 scount[]simps card[]image zero []notin[]Suc[]image [141] Overfull \hbox (1.49925pt too wide) in paragraph at lines 1952--1954 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 sfirst$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 simps$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 of P $\OML/cmm/m/it/10 ! $$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [142] Overfull \hbox (2.3468pt too wide) in paragraph at lines 2024--2027 [][] \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 sdrop$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 simps $\OMS/cmsy/m/n/10 ^^C$ \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 cases P $\OML/cmm/m/it/10 !$$\OT1/cmr/m/n/10 )$ $($\OT1/ cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ $\OMS/cmsy/m/n/10 ^^C$$^^C$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$$)$[] [143] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Overfull \hbox (28.19022pt too wide) in paragraph at lines 2129--2142 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 stakeWhile[]def LCons[]llist[]of[]stream$\OT1/cmr/m/n/ 10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 LCons[]llist[]of[]stream$\OT1/cmr/m/n/10 )$[] ) (./TLList.tex [144] [145] [146] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [147] [148] [149] [150] Overfull \hbox (3.70673pt too wide) in paragraph at lines 1175--1188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]tllist[]def cr[]tllist[]def dest$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD in-tro$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 rel[]setI$\OT1/cmr/m/n/10 )$[] [151] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. [152] Overfull \hbox (23.40169pt too wide) in paragraph at lines 1470--1483 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 cr[]tllist[]def pcr[]tllist[]def terminal[]tllis t[]of[]llist dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD$\OT 1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. [153] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [154] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. [155] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [156] [157] Overfull \hbox (49.14331pt too wide) in paragraph at lines 2439--2452 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 trans-fer$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]conv[ ]all[]lnth split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat [158] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [159] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [160] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [161] Overfull \hbox (17.64603pt too wide) in paragraph at lines 3177--3190 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set1[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3196--3209 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set2[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3215--3228 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set3[]pre[]tllist[]def rel[]set[]def [162] Overfull \hbox (22.69978pt too wide) in paragraph at lines 3313--3315 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 tllist[]all2 C B $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 unfold[]tllist IS[]TNIL1 TER-MI-NAL1 THD1 TTL1 x$\OT1/cmr/m/ n/10 )$ $($\OT1/cmr/m/it/10 unfold[]tllist Overfull \hbox (8.84482pt too wide) in paragraph at lines 3414--3427 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]fun[]def tllist[]all2[]tmap1 tllist[]all2[]t map2 elim$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]mono$\OT1/cmr/m/n/1 0 )$[] [163] [164] Overfull \hbox (6.9575pt too wide) in paragraph at lines 3655--3657 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases $\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]T Cons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 Overfull \hbox (4.40196pt too wide) in paragraph at lines 3672--3674 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases$\OT1/cmr/m/n/10 ($\OT1/cmr /m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]TC ons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 ) (./Quotient_Coinductive_List.tex [165] Overfull \hbox (13.30737pt too wide) in paragraph at lines 168--181 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]llist[]all2 symp []llist[]all2 transp[]llist[]all2$\OT1/cmr/m/n/10 )$[] [166] Overfull \hbox (52.5827pt too wide) in paragraph at lines 202--204 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 a$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1 /cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotie nt3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [167] Overfull \hbox (4.68169pt too wide) in paragraph at lines 339--352 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient[]lmap[]Abs[]Rep Quotient[]llist[]all2[]lmap[]Rep Overfull \hbox (2.09499pt too wide) in paragraph at lines 433--446 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fact lmap[]transfer$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it /10 llist[]all2[]conv[]all[]lnth lmap[]eq[]lmap[]conv[]llist[]all2 [168] Overfull \hbox (73.35773pt too wide) in paragraph at lines 515--516 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\ OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient[]lmap[]Abs[]Rep$\ OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Quotient_TLList.tex [169] Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [170] Overfull \hbox (23.27394pt too wide) in paragraph at lines 254--267 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]tllist[]all2 sym p[]tllist[]all2 transp[]tllist[]all2$\OT1/cmr/m/n/10 )$[] Overfull \hbox (55.70293pt too wide) in paragraph at lines 327--340 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ts$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/1 0 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]rep[]reflp$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotien t3[]rep[]reflp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [171] Overfull \hbox (28.84264pt too wide) in paragraph at lines 429--442 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient3[]tmap[]Abs[]Rep Quotient3[]tllist[]all2[]tmap[]tmapI Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [172] Overfull \hbox (32.54527pt too wide) in paragraph at lines 511--513 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp ad d$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]conv[]all[]tnth dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat not[]lfinite[]llength$\OT1 /cmr/m/n/10 )$[] [173] Overfull \hbox (8.50388pt too wide) in paragraph at lines 618--620 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]is[]TNilD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]tfinite1[]terminalD tllist[]all2[]thdD Overfull \hbox (49.95847pt too wide) in paragraph at lines 657--665 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 fun[]eq[]iff map[]fun[]def comp[]def Quotient3[]rel []rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it /10 Quotient3[]rel[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] Overfull \hbox (52.91345pt too wide) in paragraph at lines 693--695 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 b rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Q uotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (10.2469pt too wide) in paragraph at lines 693--695 \OT1/cmr/m/it/10 q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT 1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quoti ent3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q3$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 Quotient3[]tmap[]Abs[]Rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Coinductive.tex [174]) (./Lazy_LList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [175] [176] [177] [178] [179] [180]) (./Lazy_TLList.tex [181] Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [182] [183] [184] [185]) (./CCPO_Topology.tex [186] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. [187] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [188] [189] Overfull \hbox (9.69476pt too wide) in paragraph at lines 733--737 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] [190] Overfull \hbox (9.69476pt too wide) in paragraph at lines 758--762 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] Overfull \hbox (10.55899pt too wide) in paragraph at lines 817--819 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 intro chain[]im ageI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 le[]a$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 op $\OMS/cmsy/m/n/10 ^^T$$\OT1/cmr/m/n/10 ]$ \OT1/cmr/ m/it/10 C$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 mcont[]def monotone[]def$\OT1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. [191] [192]) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [193] [194] Overfull \hbox (10.85344pt too wide) in paragraph at lines 381--394 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq split$\OT1/cmr/m/n /10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (6.05344pt too wide) in paragraph at lines 401--414 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[]ord[]def dest$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF assms$\OT1/cmr/m/n/10 ]$$)$[] [195] Overfull \hbox (17.85112pt too wide) in paragraph at lines 518--520 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def terminal[]tllist[]of[]llist image[]ima ge$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cm r/m/it/10 rev[]image[]eqI Overfull \hbox (24.56375pt too wide) in paragraph at lines 523--525 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]upper$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/ cmr/m/it/10 blast Overfull \hbox (25.60872pt too wide) in paragraph at lines 536--538 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule contrapos []np$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \O T1/cmr/m/it/10 lprefix[]antisym chain[]lSup[]lprefix chain[]lprefix[]lSup Overfull \hbox (7.71898pt too wide) in paragraph at lines 536--538 \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def image[] image A chain[]tllist[]llist[]of[]tllist$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 rep[]eq Overfull \hbox (59.82928pt too wide) in paragraph at lines 553--555 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image chain[]lprefix[]lSup chain[]tllist[]llist[]of[]t llist [196] Overfull \hbox (83.78731pt too wide) in paragraph at lines 561--565 \OT1/cmr/m/it/10 chain[]lprefix[]lSup chain[]tllist[]llist[]of[]tllist not[]lfi nite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN iffD1$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 terminal[]tllist[]of[]llist Overfull \hbox (20.74199pt too wide) in paragraph at lines 607--609 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image not[]lfinite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN Overfull \hbox (11.60599pt too wide) in paragraph at lines 628--632 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 pre-fix \OT1/cmr/bx/n/10 have \OT1/cmr/m/it/10 lSup $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llist[]of[]tllist ` A $\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 llist[]of[]tllist xs \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lprefix[]antisym$\OT1/cmr/m/n/10 )$[ ] Overfull \hbox (24.05267pt too wide) in paragraph at lines 635--637 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\O ML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT 1/cmr/m/it/10 auto Overfull \hbox (10.06415pt too wide) in paragraph at lines 635--637 \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]tllist[]term inal$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/ it/10 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lub simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[] ord[]def$\OT1/cmr/m/n/10 )$[] [197] Overfull \hbox (10.475pt too wide) in paragraph at lines 665--667 [][] \OT1/cmr/bx/n/10 by $\OMS/cmsy/m/n/10 ^^@$$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 rule ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/ m/it/10 ccpo$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cm r/m/n/10 ]$$]$$\OML/cmm/m/it/10 ;$ Overfull \hbox (0.63309pt too wide) in paragraph at lines 692--705 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s Overfull \hbox (0.63309pt too wide) in paragraph at lines 710--723 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s [198] [199] [200] [201] Overfull \hbox (19.03722pt too wide) in paragraph at lines 1257--1260 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 chain \OT1/cmr/bx/n/10 by$ \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chain[]imageI$\OT1/cmr/m/n/10 [$\OT1/cm r/m/it/10 OF chain[]subset$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]ttlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [202] Overfull \hbox (4.28688pt too wide) in paragraph at lines 1531--1548 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT 1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF tnil$\OT1/cmr/m/ n/10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [203] Overfull \hbox (71.64563pt too wide) in paragraph at lines 1565--1583 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term tl-list$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body b$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/ 10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 fixp[]rule[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where b$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 ]$$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n /10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 fixp[]induct[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where ) (./TLList_CCPO_Examples.tex [204] [205]) (./Koenigslemma.tex [206] Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [207] Overfull \hbox (64.58913pt too wide) in paragraph at lines 233--235 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]assoc$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 metis lappend[]assoc lappend[]llist[]of[]LCons lappend[]llist[]of[]llist[] of [208] [209] [210] [211]) (./LMirror.tex [212] [213] Overfull \hbox (46.50336pt too wide) in paragraph at lines 194--196 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induction ar-bi- trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it /10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]code$\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$[$\OT1/cmr/m/it/10 symmetric$\OT1/ cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[ ]code$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$)$[] Overfull \hbox (18.66428pt too wide) in paragraph at lines 241--248 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 hide[]lams$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 no[]type s$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 add$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 c ommute epred[]llength iadd[]Suc[]right lhd[]LCons[]ltl [214] Overfull \hbox (17.3283pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 acc acc$ [] $ xs xs$ [] $$\OT1/cmr/m/n/ 10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[ ]lmirror[]aux ltl[]lmirror[]aux Overfull \hbox (61.63919pt too wide) in paragraph at lines 480--493 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases k m n rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all Overfull \hbox (4.2604pt too wide) in paragraph at lines 525--528 [][] \OT1/cmr/bx/n/10 us-ing []\OT1/cmr/m/it/10 lfinite acc[] \OT1/cmr/bx/n/ 10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 llength[]lmirror[]aux dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lfin ite[]llength[]enat$\OT1/cmr/m/n/10 )$[] [215]) (./Hamming_Stream.tex [216] [217] Overfull \hbox (14.78528pt too wide) in paragraph at lines 326--334 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (16.9785pt too wide) in paragraph at lines 343--345 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cm r/m/n/10 ($\OT1/cmr/m/it/10 1 3 4$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF mono$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m /n/10 :$ \OT1/cmr/m/it/10 F[]def lmerge[]simps Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] Overfull \hbox (11.89853pt too wide) in paragraph at lines 367--369 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono2 mono$\OT1/cmr/m/n/10 )$$+$[] Overfull \hbox (16.8158pt too wide) in paragraph at lines 427--429 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont 2mcont$\OT1/cmr/m/n/10 )$$+$[] [218] [219] Overfull \hbox (13.33519pt too wide) in paragraph at lines 704--717 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[]lmerge ltl[]lme rge not[]lnull[]conv [220] Overfull \hbox (51.39769pt too wide) in paragraph at lines 1000--1014 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 hamming[]def \OT1/cmr/bx/n/10 b y$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 ham-ming$ [] $$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]induct$\OT1/cmr/ m/n/10 )$$($\OT1/cmr/m/it/10 auto 6 6 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 in[]lset[]lmergeD$\OT1/cmr/m/n/10 )$[] Overfull \hbox (24.94225pt too wide) in paragraph at lines 1029--1034 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength ham-ming $\OT1/cm r/m/n/10 =$ \OT1/cmr/m/it/10 enat n \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/ 10 lfinite[]conv[]llength[]enat [221] Overfull \hbox (10.80869pt too wide) in paragraph at lines 1055--1057 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cmr/ m/n/10 ($\OT1/cmr/m/it/10 asm$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 hamming[]unfo ld$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 cases n$\OML/cmm/m/it/10 ;$ \OT1/cmr/m /it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ Overfull \hbox (39.67842pt too wide) in paragraph at lines 1087--1089 \OT1/cmr/m/it/10 in[]lset[]lmergeD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 s mooth[]ge[]Suc0 lsorted[]lmerge lsorted[]lmap mono-toneI ldistinct[]lmerge [222] Overfull \hbox (12.65755pt too wide) in paragraph at lines 1208--1210 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst hammin g[]unfold$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 not[]less lsorted[]lmap lsorted[]lmerge ) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype [223] Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim [224] Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL [225] Overfull \hbox (32.29482pt too wide) in paragraph at lines 239--247 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION[]def TERMINAL[]def LINEAR[]de f BRANCH[]def Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree [226] Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] Overfull \hbox (6.82832pt too wide) in paragraph at lines 406--414 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption Overfull \hbox (61.77362pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def case[]resum ption[]def Abs[]resumption[]inverse [227] Overfull \hbox (41.57692pt too wide) in paragraph at lines 515--524 [][] \OT1/cmr/m/it/10 Nit-pick$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 register[]c odatatype $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 typ $\OT1/cmr /m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$ \OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m /it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion$\OMS/cmsy/m/n/10 g$ $ \OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 const[]name case[]resump tion$\OMS/cmsy/m/n/10 g$[] [228] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [229] Overfull \hbox (10.79494pt too wide) in paragraph at lines 719--721 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule conjI str ip LINEAR[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upper$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 BRANCH[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upp er$\OT1/cmr/m/n/10 ]$ Overfull \hbox (17.23096pt too wide) in paragraph at lines 814--816 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto split$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 resumption[]corec$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 splits simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[] def Branch[]def Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [230] [231] Overfull \hbox (28.5241pt too wide) in paragraph at lines 995--998 [][] \OT1/cmr/bx/n/10 hence $[]$\OT1/cmr/m/it/10 k$\OML/cmm/m/it/10 :$ \OT1/cm r/m/it/10 ntrunc k r $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 ntrunc k r$ [] $ \OT1 /cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule Eq[]RESUMPTION[]implies []ntrunc[]equality$\OT1/cmr/m/n/10 )$[] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion [232] [233] Overfull \hbox (21.40091pt too wide) in paragraph at lines 1237--1239 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases r$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 h h$ [] $ Rep[]resumption[]constructors Eq[]RESUMPTION[]refl Overfull \hbox (89.4882pt too wide) in paragraph at lines 1284--1287 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 eq$\OT1/cmr/m/n/10 :$ $($$\OML/cm m/m/it/10 ^^U$\OT1/cmr/m/it/10 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 Rep[]resu mption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1/cmr/m/n/10 )$$)$ $=$ \OT1/c mr/m/it/10 RESUMPTION[]corec f \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 rule equals[]RESUMPTION[]corec$\OT1/cmr/m/n/10 )$[] Overfull \hbox (29.55049pt too wide) in paragraph at lines 1287--1289 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1 /cmr/m/n/10 )$$)$ $=$ \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/ cmr/m/it/10 RESUMPTION[]corec [234]) (./Coinductive_Examples.tex)) [235] (./root.aux) Package rerunfilecheck Warning: File `root.out' has changed. (rerunfilecheck) Rerun to get outlines right (rerunfilecheck) or use package `bookmark'. ) (see the transcript file for additional information) Output written on root.pdf (235 pages, 717361 bytes). Transcript written on root.log. This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty) (./isabellesym.sty) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) (./root.aux) (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (./root.out) (./root.out) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) (./root.toc [1{/var/li b/texmf/fonts/map/pdftex/updmap/pdftex.map}] [2] [3]) [4] (./session.tex (./Coinductive_Nat.tex [5] [6] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [7] Overfull \hbox (25.18492pt too wide) in paragraph at lines 655--668 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus one[]enat[]def zero[]enat[]def eSuc[]def epred[]numeral[]def Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [8] Overfull \hbox (59.08212pt too wide) in paragraph at lines 735--748 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]coexhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/ 10 case[]product enat[]coexhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 simp[ ]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus$\OT1/cmr/m/n/10 )$[] Overfull \hbox (26.72835pt too wide) in paragraph at lines 771--784 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 )$[] [9] Overfull \hbox (23.20164pt too wide) in paragraph at lines 952--969 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 bot[]enat[]def Sup[]enat[]def epred[]Max inj[ ]on[]def neq[]zero[]conv[]eSuc [10] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [11] [12] Overfull \hbox (64.72255pt too wide) in paragraph at lines 1437--1450 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y m rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all$\OML/cmm/m/it/10 ;$ [13] Overfull \hbox (22.26717pt too wide) in paragraph at lines 1545--1558 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m x y rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (22.99493pt too wide) in paragraph at lines 1563--1576 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m k rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (53.3571pt too wide) in paragraph at lines 1625--1627 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Sup[]enat[]def Max[]enat[]minus1 finite[]less Than[]enat[]iff enat[]diff[]cancel[]left [14] [15] Overfull \hbox (11.05505pt too wide) in paragraph at lines 1990--2003 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]eadd1 mcont[]eadd2 [16] Overfull \hbox (6.50609pt too wide) in paragraph at lines 2143--2145 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule finite[ ]imageD$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 inj[]onI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 max[]de f split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [17] Overfull \hbox (52.5326pt too wide) in paragraph at lines 2239--2252 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]max[]enat1 mcont[]max[]enat2 [18] [19]) (./Coinductive_List.tex [20] [21] [22] [23] [24] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. [25] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [26] [27] [28] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [29] [30] Overfull \hbox (16.47273pt too wide) in paragraph at lines 1960--1962 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys zs$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv LCons[]lprefix[]conv$\OML/cmm/m/it/10 ;$ [31] Overfull \hbox (1.58864pt too wide) in paragraph at lines 2103--2116 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSup$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 lprefix[]lhdD in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]e quality$\OT1/cmr/m/n/10 )$[] [32] Overfull \hbox (24.56723pt too wide) in paragraph at lines 2175--2188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 expand$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto si mp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image lhd[]lSup exI LCons[]im age[]Int[]not[]lnull Overfull \hbox (14.04483pt too wide) in paragraph at lines 2290--2293 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 ?LCons \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/i t/10 the[]equality dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lprefix[]lhdD in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]image[]eqI$\OT1/cmr/m/n/10 )$[] [33] [34] [35] [36] Overfull \hbox (0.19804pt too wide) in paragraph at lines 2834--2847 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF lnil$\OT1/cmr/m/n/ 10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (24.52327pt too wide) in paragraph at lines 2874--2887 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 monotone[]if[]bot$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 f$\OT1/cmr/m/n/10 =$$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it /10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 f $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 lhd xs$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 ltl xs$\OT1/cmr/m/n/10 )$ \OT1 /cmr/m/it/10 xs \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 bound$\OT1/cmr/m/n/10 =$\ OT1/cmr/m/it/10 LNil$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto Overfull \hbox (2.5006pt too wide) in paragraph at lines 2874--2887 \OT1/cmr/m/it/10 4 3 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 split simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv LCons[]lprefix[]conv dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mo no-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.96495pt too wide) in paragraph at lines 2915--2919 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 ob-tain \OT1/cm r/m/it/10 x xs \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 LCons x xs $\OMS/cmsy/m/ n/10 2$ \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv$\OT1 /cmr/m/n/10 )$[] Overfull \hbox (3.45793pt too wide) in paragraph at lines 2922--2924 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force dest$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF cha in$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 LCons[]lprefix[]conv lprefix[]LCons[]conv [37] Overfull \hbox (11.3537pt too wide) in paragraph at lines 3014--3036 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term llist$\OML/c mm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @ $$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 fixp[]rule[]uc$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$ \OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]strong[]in duct[]uc$\OMS/cmsy/m/n/10 g$ Overfull \hbox (10.92476pt too wide) in paragraph at lines 3050--3058 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [38] Overfull \hbox (10.92476pt too wide) in paragraph at lines 3225--3233 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [39] Overfull \hbox (11.56499pt too wide) in paragraph at lines 3404--3406 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSu p$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 dest$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ] $ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]equality$ \OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ [40] [41] [42] [43] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [44] Overfull \hbox (16.78535pt too wide) in paragraph at lines 3905--3907 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs$ [] $ rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]induct$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Nil lappend[]llis t[]of[]llist[]of$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ] $ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [45] [46] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Overfull \hbox (15.20331pt too wide) in paragraph at lines 4386--4399 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 epred[]iadd1 [47] [48] Overfull \hbox (10.92476pt too wide) in paragraph at lines 4665--4673 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (18.88669pt too wide) in paragraph at lines 4677--4679 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 subst $\OT1/cmr/m /n/10 ($\OT1/cmr/m/it/10 1 2 3$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lfp$\OML/cmm /m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (17.23381pt too wide) in paragraph at lines 4692--4705 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/ 10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Overfull \hbox (19.53375pt too wide) in paragraph at lines 4711--4728 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it /10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [49] Overfull \hbox (17.11995pt too wide) in paragraph at lines 4940--4953 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\ OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff [50] [51] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5331--5339 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [52] [53] [54] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5786--5794 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [55] [56] [57] [58] Overfull \hbox (25.67209pt too wide) in paragraph at lines 6689--6693 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 LCons \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/1 0 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 )$$($\OT1/cm r/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]Suc[]right$\O T1/cmr/m/n/10 )$[] [59] Overfull \hbox (68.23685pt too wide) in paragraph at lines 6786--6790 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Cons \OT1/cmr/bx/n/10 thus \OT1/cm r/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (27.84201pt too wide) in paragraph at lines 6882--6895 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldrop[]LCons iadd[]Suc[]righ t split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it /10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.39761pt too wide) in paragraph at lines 6900--6917 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltake[]LCons ldrop[]LCons sp lit$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [60] [61] [62] Overfull \hbox (1.621pt too wide) in paragraph at lines 7327--7330 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ex I$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 = $\OT1/cmr/m/it/10 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/1 0 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (19.0108pt too wide) in paragraph at lines 7336--7338 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 wh ere \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc n \OT1/cmr/bx/n/1 0 for \OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ileI1 simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] [63] Overfull \hbox (28.40157pt too wide) in paragraph at lines 7638--7651 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis eSuc[]enat eSu c[]plus[]1 ltake[]plus[]conv[]lappend ldrop[]enat ldropn[]Suc[]conv[]ldropn [64] [65] [66] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [67] Overfull \hbox (5.19078pt too wide) in paragraph at lines 8236--8249 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def lnull[]d ef neq[]LNil[]conv [68] [69] Overfull \hbox (4.94086pt too wide) in paragraph at lines 8503--8516 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 prefix[]def lprefix[]conv[]lappend$\OT1/cmr/m/n/1 0 )$$($\OT1/cmr/m/it/10 metis lfinite[]lappend lfinite[]llist[]of Overfull \hbox (21.38031pt too wide) in paragraph at lines 8611--8616 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lSup A$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 enat n \OT1/c mr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 lfinite[]conv[]llength[]enat Overfull \hbox (2.40771pt too wide) in paragraph at lines 8620--8623 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 fi-nite $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 llength ` A$\OT1/cmr/m/n/10 )$ \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ( $\OT1/cmr/m/it/10 rule finite[]subset$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 sim p add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 finite[]lessThan[]enat[]iff$\OT1/cmr/ m/n/10 )$[] [70] Overfull \hbox (13.92545pt too wide) in paragraph at lines 8799--8812 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llcp[]eq[]0[]iff epred[]llcp [71] Overfull \hbox (10.21999pt too wide) in paragraph at lines 8818--8831 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 llcp[]eq[]0[]iff Overfull \hbox (14.39069pt too wide) in paragraph at lines 8836--8849 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis add[]0[]right lappend[]LNil2 llcp[]LNil1 llcp[]lappend[]same lprefix[]conv[]lappend$\OT1/cmr /m/n/10 )$[] Overfull \hbox (52.74213pt too wide) in paragraph at lines 8897--8899 \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/ cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 iadd[]Suc[]right zero []enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[ ] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [72] Overfull \hbox (5.10889pt too wide) in paragraph at lines 9073--9086 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff Overfull \hbox (14.78528pt too wide) in paragraph at lines 9140--9148 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [73] Overfull \hbox (2.44716pt too wide) in paragraph at lines 9295--9298 [][] \OT1/cmr/bx/n/10 thus \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr /m/n/10 ($\OT1/cmr/m/it/10 cases ys n rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 case[]product co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/1 0 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr/m/it/10 simp[]all[] [74] [75] [76] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9748--9761 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9767--9780 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9788--9805 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [77] Overfull \hbox (10.92476pt too wide) in paragraph at lines 9859--9867 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (0.88739pt too wide) in paragraph at lines 9893--9906 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr /m/it/10 simp[] Overfull \hbox (3.18733pt too wide) in paragraph at lines 9912--9925 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cm r/m/it/10 simp[] [78] [79] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset Overfull \hbox (23.46579pt too wide) in paragraph at lines 10431--10444 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv [80] [81] Overfull \hbox (4.60457pt too wide) in paragraph at lines 10598--10606 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 llength[]ltakeWhile[]all$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 llen gth[]eq[]infty[]conv[]lfinite$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1 /cmr/m/n/10 ]$[] Overfull \hbox (34.96571pt too wide) in paragraph at lines 10694--10707 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n /10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [82] Overfull \hbox (6.35873pt too wide) in paragraph at lines 10905--10918 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]eq[]infty[]conv[]l finite lfinite[]ltakeWhile$\OT1/cmr/m/n/10 )$[] Overfull \hbox (43.52377pt too wide) in paragraph at lines 10925--10938 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]ldrop llength[]lta keWhile[]all ltakeWhile[]all[]conv [83] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [84] Overfull \hbox (31.74066pt too wide) in paragraph at lines 11315--11317 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 step llist[]all2[]llengthD [85] Overfull \hbox (25.92279pt too wide) in paragraph at lines 11331--11333 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases lnull xs $\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 step simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cm r/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lnth[ ]0[]conv[]lhd$\OT1/cmr/m/n/10 )$[] [86] Overfull \hbox (37.6261pt too wide) in paragraph at lines 11639--11644 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth ys n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 ltake $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llength xs$\OT 1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 n \OT1/ cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lnth[]ltake$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (4.15424pt too wide) in paragraph at lines 11644--11649 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lappend xs xs$ [] $$\OT1 /cmr/m/n/10 )$ \OT1/cmr/m/it/10 n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth xs n \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 lnth[]lappend1$\OT1/cmr/m/n/10 )$[] [87] Overfull \hbox (15.4463pt too wide) in paragraph at lines 11688--11690 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 neq[]LNil[]conv lnul l[]def LNil[]eq[]lmap Overfull \hbox (24.38661pt too wide) in paragraph at lines 11696--11698 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lnullD llis t[]all2[]lhdD llist[]all2[]ltlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (7.40894pt too wide) in paragraph at lines 11742--11749 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [88] Overfull \hbox (12.14566pt too wide) in paragraph at lines 11911--11913 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image dest$\OT1/cmr/m/n/10 :$ \ OT1/cmr/m/it/10 Y llist[]all2[]lnullD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 rev[]image[]eqI$\OT1/cmr/m/n/10 )$$+$[] [89] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. [90] Overfull \hbox (18.37143pt too wide) in paragraph at lines 12252--12256 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Suc \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x s$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$ \OT1/cmr/m/it/10 llast[]LCons$\OT1/cmr/m/n/10 )$[] [91] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [92] Overfull \hbox (5.61943pt too wide) in paragraph at lines 12468--12472 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chain[]lprefix[]ltl chain in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldistinct[]ltlI Overfull \hbox (17.75882pt too wide) in paragraph at lines 12506--12508 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ldistinct[]lSup chain[]imageI mcont[ ]monoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [93] [94] Overfull \hbox (0.21182pt too wide) in paragraph at lines 12872--12889 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv des t$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lset[]lzipD2$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [95] Overfull \hbox (3.13603pt too wide) in paragraph at lines 13020--13025 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 us -ing \OT1/cmr/m/it/10 chain sorted \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]ltl lsorted[]ltlI$\OT1/cmr/m/n/10 )$[] [96] Overfull \hbox (11.49773pt too wide) in paragraph at lines 13106--13108 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lsorted[]lSup chain[]imageI mcont[]m onoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (12.42061pt too wide) in paragraph at lines 13121--13134 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 admissibleI$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 aut o dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lsorted[]lprefixD$\OT1/cmr/m/n/10 [$ \OT1/cmr/m/it/10 rotated$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]lSup$\OT1/cmr/m/n/10 )$[] Overfull \hbox (4.57834pt too wide) in paragraph at lines 13157--13170 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct n ar-bi-trary $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 f astforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldropn[]Suc lsorted[]LCon s$ [] $ ldropn[]lnull [97] Overfull \hbox (1.39157pt too wide) in paragraph at lines 13303--13310 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lsorted[]coinduct$ [] $$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mon o-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [98] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [99] [100] [101] [102] [103] [104] [105] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [106] Overfull \hbox (5.09007pt too wide) in paragraph at lines 14626--14639 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 drule eq[]LConsD$\OT 1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m /it/10 exI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltl[]lfilter o[]def ldr opWhile[]eq[]LNil[]iff [107] [108] [109] [110] Overfull \hbox (14.26587pt too wide) in paragraph at lines 15252--15254 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]snocL1[]conv[]LCons2$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 symmetric$\OML/cmm/m/it/10 ;$ \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 lappend [111] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [112] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [113] [114] [115] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [116] [117] Overfull \hbox (13.61642pt too wide) in paragraph at lines 16286--16290 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 concat[]xss$ [] $ nth[]n \OT 1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 xss \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lnth[]lappe nd2 lappend[]lnull1$\OT1/cmr/m/n/10 )$[] [118] Overfull \hbox (1.33876pt too wide) in paragraph at lines 16330--16332 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/ cmr/m/n/10 ($\OT1/cmr/m/it/10 1 2$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 atLeast0L essThan$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$$($\O T1/cmr/m/it/10 subst sum[]add[]nat[]ivl$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 si mp[]all$\OT1/cmr/m/n/10 )$[] [119] [120] Overfull \hbox (4.77174pt too wide) in paragraph at lines 16574--16576 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 lfilter[]eq[]LConsD$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF []LCons x xs $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lfi l-ter $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 xs$\OML/cmm/m/i t/10 :$ $\OMS/cmsy/m/n/10 :$ \OT1/cmr/m/it/10 lnull xs$\OT1/cmr/m/n/10 )$ \OT1/ cmr/m/it/10 xss[]$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$]$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [121] [122] [123] [124] [125] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [126] [127] [128] [129] Overfull \hbox (11.00165pt too wide) in paragraph at lines 18136--18149 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set1[]pre[]llist[]def rel[]set[]def Overfull \hbox (11.00165pt too wide) in paragraph at lines 18155--18168 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set2[]pre[]llist[]def rel[]set[]def [130] [131] [132]) (./Coinductive_List_Prefix.tex [133] [134] Overfull \hbox (17.24495pt too wide) in paragraph at lines 330--336 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 Sup[]llist[]def less[]eq[]llist[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 abs[]def$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]upper llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]least$\OT1/cmr/m/n/10 )$[] ) (./Coinductive_Stream.tex [135] [136] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [137] [138] [139] [140] Overfull \hbox (1.53853pt too wide) in paragraph at lines 1044--1057 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]stream[]def cr[]stream[]def in-tro$\OT1/ cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 rel[]funI rel-comppI rel[]setI [141] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. [142] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [143] Overfull \hbox (6.55463pt too wide) in paragraph at lines 1618--1624 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 bot[]enat[]def in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 admiss ible[]all admissible[]imp admissible[]eq[]mcontI Overfull \hbox (32.81557pt too wide) in paragraph at lines 1702--1707 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 step \OT1/cmr/bx/n/10 un-fol d-ing \OT1/cmr/m/it/10 eq \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 scount[]simps card[]image zero []notin[]Suc[]image [144] Overfull \hbox (1.49925pt too wide) in paragraph at lines 1952--1954 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 sfirst$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 simps$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 of P $\OML/cmm/m/it/10 ! $$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [145] Overfull \hbox (2.3468pt too wide) in paragraph at lines 2024--2027 [][] \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 sdrop$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 simps $\OMS/cmsy/m/n/10 ^^C$ \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 cases P $\OML/cmm/m/it/10 !$$\OT1/cmr/m/n/10 )$ $($\OT1/ cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ $\OMS/cmsy/m/n/10 ^^C$$^^C$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$$)$[] [146] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Overfull \hbox (28.19022pt too wide) in paragraph at lines 2129--2142 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 stakeWhile[]def LCons[]llist[]of[]stream$\OT1/cmr/m/n/ 10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 LCons[]llist[]of[]stream$\OT1/cmr/m/n/10 )$[] ) (./TLList.tex [147] [148] [149] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [150] [151] [152] [153] Overfull \hbox (3.70673pt too wide) in paragraph at lines 1175--1188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]tllist[]def cr[]tllist[]def dest$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD in-tro$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 rel[]setI$\OT1/cmr/m/n/10 )$[] [154] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. [155] Overfull \hbox (23.40169pt too wide) in paragraph at lines 1470--1483 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 cr[]tllist[]def pcr[]tllist[]def terminal[]tllis t[]of[]llist dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD$\OT 1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. [156] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [157] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. [158] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [159] [160] Overfull \hbox (49.14331pt too wide) in paragraph at lines 2439--2452 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 trans-fer$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]conv[ ]all[]lnth split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat [161] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [162] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [163] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [164] Overfull \hbox (17.64603pt too wide) in paragraph at lines 3177--3190 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set1[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3196--3209 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set2[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3215--3228 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set3[]pre[]tllist[]def rel[]set[]def [165] Overfull \hbox (22.69978pt too wide) in paragraph at lines 3313--3315 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 tllist[]all2 C B $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 unfold[]tllist IS[]TNIL1 TER-MI-NAL1 THD1 TTL1 x$\OT1/cmr/m/ n/10 )$ $($\OT1/cmr/m/it/10 unfold[]tllist Overfull \hbox (8.84482pt too wide) in paragraph at lines 3414--3427 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]fun[]def tllist[]all2[]tmap1 tllist[]all2[]t map2 elim$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]mono$\OT1/cmr/m/n/1 0 )$[] [166] [167] Overfull \hbox (6.9575pt too wide) in paragraph at lines 3655--3657 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases $\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]T Cons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 Overfull \hbox (4.40196pt too wide) in paragraph at lines 3672--3674 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases$\OT1/cmr/m/n/10 ($\OT1/cmr /m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]TC ons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 ) (./Quotient_Coinductive_List.tex [168] Overfull \hbox (13.30737pt too wide) in paragraph at lines 168--181 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]llist[]all2 symp []llist[]all2 transp[]llist[]all2$\OT1/cmr/m/n/10 )$[] [169] Overfull \hbox (52.5827pt too wide) in paragraph at lines 202--204 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 a$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1 /cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotie nt3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [170] Overfull \hbox (4.68169pt too wide) in paragraph at lines 339--352 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient[]lmap[]Abs[]Rep Quotient[]llist[]all2[]lmap[]Rep Overfull \hbox (2.09499pt too wide) in paragraph at lines 433--446 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fact lmap[]transfer$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it /10 llist[]all2[]conv[]all[]lnth lmap[]eq[]lmap[]conv[]llist[]all2 [171] Overfull \hbox (73.35773pt too wide) in paragraph at lines 515--516 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\ OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient[]lmap[]Abs[]Rep$\ OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Quotient_TLList.tex [172] Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [173] Overfull \hbox (23.27394pt too wide) in paragraph at lines 254--267 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]tllist[]all2 sym p[]tllist[]all2 transp[]tllist[]all2$\OT1/cmr/m/n/10 )$[] Overfull \hbox (55.70293pt too wide) in paragraph at lines 327--340 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ts$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/1 0 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]rep[]reflp$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotien t3[]rep[]reflp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [174] Overfull \hbox (28.84264pt too wide) in paragraph at lines 429--442 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient3[]tmap[]Abs[]Rep Quotient3[]tllist[]all2[]tmap[]tmapI Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [175] Overfull \hbox (32.54527pt too wide) in paragraph at lines 511--513 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp ad d$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]conv[]all[]tnth dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat not[]lfinite[]llength$\OT1 /cmr/m/n/10 )$[] [176] Overfull \hbox (8.50388pt too wide) in paragraph at lines 618--620 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]is[]TNilD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]tfinite1[]terminalD tllist[]all2[]thdD Overfull \hbox (49.95847pt too wide) in paragraph at lines 657--665 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 fun[]eq[]iff map[]fun[]def comp[]def Quotient3[]rel []rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it /10 Quotient3[]rel[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] Overfull \hbox (52.91345pt too wide) in paragraph at lines 693--695 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 b rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Q uotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (10.2469pt too wide) in paragraph at lines 693--695 \OT1/cmr/m/it/10 q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT 1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quoti ent3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q3$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 Quotient3[]tmap[]Abs[]Rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Coinductive.tex [177]) (./Lazy_LList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [178] [179] [180] [181] [182] [183]) (./Lazy_TLList.tex [184] Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [185] [186] [187] [188]) (./CCPO_Topology.tex [189] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. [190] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [191] [192] Overfull \hbox (9.69476pt too wide) in paragraph at lines 733--737 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] [193] Overfull \hbox (9.69476pt too wide) in paragraph at lines 758--762 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] Overfull \hbox (10.55899pt too wide) in paragraph at lines 817--819 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 intro chain[]im ageI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 le[]a$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 op $\OMS/cmsy/m/n/10 ^^T$$\OT1/cmr/m/n/10 ]$ \OT1/cmr/ m/it/10 C$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 mcont[]def monotone[]def$\OT1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. [194] [195]) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [196] [197] Overfull \hbox (10.85344pt too wide) in paragraph at lines 381--394 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq split$\OT1/cmr/m/n /10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (6.05344pt too wide) in paragraph at lines 401--414 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[]ord[]def dest$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF assms$\OT1/cmr/m/n/10 ]$$)$[] [198] Overfull \hbox (17.85112pt too wide) in paragraph at lines 518--520 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def terminal[]tllist[]of[]llist image[]ima ge$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cm r/m/it/10 rev[]image[]eqI Overfull \hbox (24.56375pt too wide) in paragraph at lines 523--525 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]upper$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/ cmr/m/it/10 blast Overfull \hbox (25.60872pt too wide) in paragraph at lines 536--538 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule contrapos []np$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \O T1/cmr/m/it/10 lprefix[]antisym chain[]lSup[]lprefix chain[]lprefix[]lSup Overfull \hbox (7.71898pt too wide) in paragraph at lines 536--538 \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def image[] image A chain[]tllist[]llist[]of[]tllist$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 rep[]eq Overfull \hbox (59.82928pt too wide) in paragraph at lines 553--555 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image chain[]lprefix[]lSup chain[]tllist[]llist[]of[]t llist [199] Overfull \hbox (83.78731pt too wide) in paragraph at lines 561--565 \OT1/cmr/m/it/10 chain[]lprefix[]lSup chain[]tllist[]llist[]of[]tllist not[]lfi nite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN iffD1$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 terminal[]tllist[]of[]llist Overfull \hbox (20.74199pt too wide) in paragraph at lines 607--609 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image not[]lfinite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN Overfull \hbox (11.60599pt too wide) in paragraph at lines 628--632 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 pre-fix \OT1/cmr/bx/n/10 have \OT1/cmr/m/it/10 lSup $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llist[]of[]tllist ` A $\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 llist[]of[]tllist xs \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lprefix[]antisym$\OT1/cmr/m/n/10 )$[ ] Overfull \hbox (24.05267pt too wide) in paragraph at lines 635--637 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\O ML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT 1/cmr/m/it/10 auto Overfull \hbox (10.06415pt too wide) in paragraph at lines 635--637 \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]tllist[]term inal$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/ it/10 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lub simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[] ord[]def$\OT1/cmr/m/n/10 )$[] [200] Overfull \hbox (10.475pt too wide) in paragraph at lines 665--667 [][] \OT1/cmr/bx/n/10 by $\OMS/cmsy/m/n/10 ^^@$$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 rule ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/ m/it/10 ccpo$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cm r/m/n/10 ]$$]$$\OML/cmm/m/it/10 ;$ Overfull \hbox (0.63309pt too wide) in paragraph at lines 692--705 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s Overfull \hbox (0.63309pt too wide) in paragraph at lines 710--723 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s [201] [202] [203] [204] Overfull \hbox (19.03722pt too wide) in paragraph at lines 1257--1260 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 chain \OT1/cmr/bx/n/10 by$ \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chain[]imageI$\OT1/cmr/m/n/10 [$\OT1/cm r/m/it/10 OF chain[]subset$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]ttlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [205] Overfull \hbox (4.28688pt too wide) in paragraph at lines 1531--1548 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT 1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF tnil$\OT1/cmr/m/ n/10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [206] Overfull \hbox (71.64563pt too wide) in paragraph at lines 1565--1583 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term tl-list$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body b$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/ 10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 fixp[]rule[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where b$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 ]$$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n /10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 fixp[]induct[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where ) (./TLList_CCPO_Examples.tex [207] [208]) (./Koenigslemma.tex [209] Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [210] Overfull \hbox (64.58913pt too wide) in paragraph at lines 233--235 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]assoc$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 metis lappend[]assoc lappend[]llist[]of[]LCons lappend[]llist[]of[]llist[] of [211] [212] [213] [214]) (./LMirror.tex [215] [216] Overfull \hbox (46.50336pt too wide) in paragraph at lines 194--196 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induction ar-bi- trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it /10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]code$\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$[$\OT1/cmr/m/it/10 symmetric$\OT1/ cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[ ]code$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$)$[] Overfull \hbox (18.66428pt too wide) in paragraph at lines 241--248 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 hide[]lams$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 no[]type s$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 add$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 c ommute epred[]llength iadd[]Suc[]right lhd[]LCons[]ltl [217] Overfull \hbox (17.3283pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 acc acc$ [] $ xs xs$ [] $$\OT1/cmr/m/n/ 10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[ ]lmirror[]aux ltl[]lmirror[]aux Overfull \hbox (61.63919pt too wide) in paragraph at lines 480--493 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases k m n rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all Overfull \hbox (4.2604pt too wide) in paragraph at lines 525--528 [][] \OT1/cmr/bx/n/10 us-ing []\OT1/cmr/m/it/10 lfinite acc[] \OT1/cmr/bx/n/ 10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 llength[]lmirror[]aux dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lfin ite[]llength[]enat$\OT1/cmr/m/n/10 )$[] [218]) (./Hamming_Stream.tex [219] [220] Overfull \hbox (14.78528pt too wide) in paragraph at lines 326--334 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (16.9785pt too wide) in paragraph at lines 343--345 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cm r/m/n/10 ($\OT1/cmr/m/it/10 1 3 4$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF mono$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m /n/10 :$ \OT1/cmr/m/it/10 F[]def lmerge[]simps Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] Overfull \hbox (11.89853pt too wide) in paragraph at lines 367--369 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono2 mono$\OT1/cmr/m/n/10 )$$+$[] Overfull \hbox (16.8158pt too wide) in paragraph at lines 427--429 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont 2mcont$\OT1/cmr/m/n/10 )$$+$[] [221] [222] Overfull \hbox (13.33519pt too wide) in paragraph at lines 704--717 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[]lmerge ltl[]lme rge not[]lnull[]conv [223] Overfull \hbox (51.39769pt too wide) in paragraph at lines 1000--1014 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 hamming[]def \OT1/cmr/bx/n/10 b y$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 ham-ming$ [] $$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]induct$\OT1/cmr/ m/n/10 )$$($\OT1/cmr/m/it/10 auto 6 6 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 in[]lset[]lmergeD$\OT1/cmr/m/n/10 )$[] Overfull \hbox (24.94225pt too wide) in paragraph at lines 1029--1034 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength ham-ming $\OT1/cm r/m/n/10 =$ \OT1/cmr/m/it/10 enat n \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/ 10 lfinite[]conv[]llength[]enat [224] Overfull \hbox (10.80869pt too wide) in paragraph at lines 1055--1057 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cmr/ m/n/10 ($\OT1/cmr/m/it/10 asm$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 hamming[]unfo ld$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 cases n$\OML/cmm/m/it/10 ;$ \OT1/cmr/m /it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ Overfull \hbox (39.67842pt too wide) in paragraph at lines 1087--1089 \OT1/cmr/m/it/10 in[]lset[]lmergeD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 s mooth[]ge[]Suc0 lsorted[]lmerge lsorted[]lmap mono-toneI ldistinct[]lmerge [225] Overfull \hbox (12.65755pt too wide) in paragraph at lines 1208--1210 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst hammin g[]unfold$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 not[]less lsorted[]lmap lsorted[]lmerge ) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype [226] Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim [227] Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL [228] Overfull \hbox (32.29482pt too wide) in paragraph at lines 239--247 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION[]def TERMINAL[]def LINEAR[]de f BRANCH[]def Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree [229] Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] Overfull \hbox (6.82832pt too wide) in paragraph at lines 406--414 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption Overfull \hbox (61.77362pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def case[]resum ption[]def Abs[]resumption[]inverse [230] Overfull \hbox (41.57692pt too wide) in paragraph at lines 515--524 [][] \OT1/cmr/m/it/10 Nit-pick$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 register[]c odatatype $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 typ $\OT1/cmr /m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$ \OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m /it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion$\OMS/cmsy/m/n/10 g$ $ \OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 const[]name case[]resump tion$\OMS/cmsy/m/n/10 g$[] [231] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [232] Overfull \hbox (10.79494pt too wide) in paragraph at lines 719--721 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule conjI str ip LINEAR[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upper$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 BRANCH[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upp er$\OT1/cmr/m/n/10 ]$ Overfull \hbox (17.23096pt too wide) in paragraph at lines 814--816 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto split$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 resumption[]corec$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 splits simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[] def Branch[]def Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [233] [234] Overfull \hbox (28.5241pt too wide) in paragraph at lines 995--998 [][] \OT1/cmr/bx/n/10 hence $[]$\OT1/cmr/m/it/10 k$\OML/cmm/m/it/10 :$ \OT1/cm r/m/it/10 ntrunc k r $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 ntrunc k r$ [] $ \OT1 /cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule Eq[]RESUMPTION[]implies []ntrunc[]equality$\OT1/cmr/m/n/10 )$[] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion [235] [236] Overfull \hbox (21.40091pt too wide) in paragraph at lines 1237--1239 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases r$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 h h$ [] $ Rep[]resumption[]constructors Eq[]RESUMPTION[]refl Overfull \hbox (89.4882pt too wide) in paragraph at lines 1284--1287 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 eq$\OT1/cmr/m/n/10 :$ $($$\OML/cm m/m/it/10 ^^U$\OT1/cmr/m/it/10 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 Rep[]resu mption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1/cmr/m/n/10 )$$)$ $=$ \OT1/c mr/m/it/10 RESUMPTION[]corec f \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 rule equals[]RESUMPTION[]corec$\OT1/cmr/m/n/10 )$[] Overfull \hbox (29.55049pt too wide) in paragraph at lines 1287--1289 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1 /cmr/m/n/10 )$$)$ $=$ \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/ cmr/m/it/10 RESUMPTION[]corec [237]) (./Coinductive_Examples.tex)) [238] (./root.aux) ) (see the transcript file for additional information) Output written on root.pdf (238 pages, 736876 bytes). Transcript written on root.log. This is pdfTeX, Version 3.14159265-2.6-1.40.16 (TeX Live 2015/Debian) (preloaded format=pdflatex) restricted \write18 enabled. entering extended mode LaTeX2e <2016/02/01> Babel <3.9q> and hyphenation patterns for 81 language(s) loaded. (./root.tex (/usr/share/texlive/texmf-dist/tex/latex/base/article.cls Document Class: article 2014/09/29 v1.4h Standard LaTeX document class (/usr/share/texlive/texmf-dist/tex/latex/base/size11.clo)) (./isabelle.sty (./comment.sty Excluding comment 'comment') Including comment 'isadelimtheory' Including comment 'isatagtheory' Including comment 'isadelimproof' Including comment 'isatagproof' Including comment 'isadelimML' Including comment 'isatagML' Including comment 'isadelimvisible' Including comment 'isatagvisible' Excluding comment 'isadeliminvisible' Excluding comment 'isataginvisible') (./isabelletags.sty) (./isabellesym.sty) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/stmaryrd.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsmath.sty For additional information on amsmath, use the `?' option. (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amstext.sty (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsgen.sty)) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsbsy.sty) (/usr/share/texlive/texmf-dist/tex/latex/amsmath/amsopn.sty)) (./pdfsetup.sty (/usr/share/texlive/texmf-dist/tex/latex/graphics/color.sty (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/color.cfg) (/usr/share/texlive/texmf-dist/tex/latex/pdftex-def/pdftex.def (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/infwarerr.sty) (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/ltxcmds.sty)))) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-hyperref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/hobsub-generic.sty)) (/usr/share/texlive/texmf-dist/tex/latex/graphics/keyval.sty) (/usr/share/texlive/texmf-dist/tex/generic/ifxetex/ifxetex.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/auxhook.sty) (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/kvoptions.sty) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/pd1enc.def) (/usr/share/texlive/texmf-dist/tex/latex/latexconfig/hyperref.cfg) (/usr/share/texlive/texmf-dist/tex/latex/url/url.sty)) Package hyperref Message: Driver (autodetected): hpdftex. (/usr/share/texlive/texmf-dist/tex/latex/hyperref/hpdftex.def (/usr/share/texlive/texmf-dist/tex/latex/oberdiek/rerunfilecheck.sty)) (./root.aux) (/usr/share/texlive/texmf-dist/tex/context/base/supp-pdf.mkii [Loading MPS to PDF converter (version 2006.09.02).] ) (/usr/share/texlive/texmf-dist/tex/latex/hyperref/nameref.sty (/usr/share/texlive/texmf-dist/tex/generic/oberdiek/gettitlestring.sty)) (./root.out) (./root.out) (/usr/share/texlive/texmf-dist/tex/latex/stmaryrd/Ustmry.fd) (/usr/share/texlive/texmf-dist/tex/latex/base/omscmr.fd) (./root.toc [1{/var/li b/texmf/fonts/map/pdftex/updmap/pdftex.map}] [2] [3]) [4] (./session.tex (./Coinductive_Nat.tex [5] [6] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 479. [7] Overfull \hbox (25.18492pt too wide) in paragraph at lines 655--668 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus one[]enat[]def zero[]enat[]def eSuc[]def epred[]numeral[]def Overfull \hbox (19.62083pt too wide) in paragraph at lines 671--673 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 epred[]simps $\OT1/cmr/m/n/10 =$ \ OT1/cmr/m/it/10 epred[]0 epred[]1 epred[]numeral epred[]eSuc epred[]Infty epred []enat[] [8] Overfull \hbox (59.08212pt too wide) in paragraph at lines 735--748 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]coexhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/ 10 case[]product enat[]coexhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 simp[ ]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 epred[]conv[]minus$\OT1/cmr/m/n/10 )$[] Overfull \hbox (26.72835pt too wide) in paragraph at lines 771--784 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y rule$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 )$[] [9] Overfull \hbox (23.20164pt too wide) in paragraph at lines 952--969 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 bot[]enat[]def Sup[]enat[]def epred[]Max inj[ ]on[]def neq[]zero[]conv[]eSuc [10] Overfull \hbox (4.53096pt too wide) in paragraph at lines 1169--1171 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 enat[]leI $\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Leenat$\ OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Leenat zero eSuc$\OT1/cmr/ m/n/10 ]$$:$[] [11] [12] Overfull \hbox (64.72255pt too wide) in paragraph at lines 1437--1450 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x y m rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all$\OML/cmm/m/it/10 ;$ [13] Overfull \hbox (22.26717pt too wide) in paragraph at lines 1545--1558 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m x y rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (22.99493pt too wide) in paragraph at lines 1563--1576 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n m k rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$ Overfull \hbox (53.3571pt too wide) in paragraph at lines 1625--1627 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Sup[]enat[]def Max[]enat[]minus1 finite[]less Than[]enat[]iff enat[]diff[]cancel[]left [14] [15] Overfull \hbox (11.05505pt too wide) in paragraph at lines 1990--2003 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]eadd1 mcont[]eadd2 [16] Overfull \hbox (6.50609pt too wide) in paragraph at lines 2143--2145 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule finite[ ]imageD$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 inj[]onI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 max[]de f split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [17] Overfull \hbox (52.5326pt too wide) in paragraph at lines 2239--2252 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 best in-tro$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont2mcon t$ [] $$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF complete[]lattice[]ccpo$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 mcont[]max[]enat1 mcont[]max[]enat2 [18] [19]) (./Coinductive_List.tex [20] [21] [22] [23] [24] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 863. [25] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 992. [26] [27] [28] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1458. [29] [30] Overfull \hbox (16.47273pt too wide) in paragraph at lines 1960--1962 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys zs$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv LCons[]lprefix[]conv$\OML/cmm/m/it/10 ;$ [31] Overfull \hbox (1.58864pt too wide) in paragraph at lines 2103--2116 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSup$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 lprefix[]lhdD in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]e quality$\OT1/cmr/m/n/10 )$[] [32] Overfull \hbox (24.56723pt too wide) in paragraph at lines 2175--2188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 expand$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto si mp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image lhd[]lSup exI LCons[]im age[]Int[]not[]lnull Overfull \hbox (14.04483pt too wide) in paragraph at lines 2290--2293 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 ?LCons \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/i t/10 the[]equality dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lprefix[]lhdD in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]image[]eqI$\OT1/cmr/m/n/10 )$[] [33] [34] [35] [36] Overfull \hbox (0.19804pt too wide) in paragraph at lines 2834--2847 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF lnil$\OT1/cmr/m/n/ 10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (24.52327pt too wide) in paragraph at lines 2874--2887 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 monotone[]if[]bot$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 f$\OT1/cmr/m/n/10 =$$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it /10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 f $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 lhd xs$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 ltl xs$\OT1/cmr/m/n/10 )$ \OT1 /cmr/m/it/10 xs \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 bound$\OT1/cmr/m/n/10 =$\ OT1/cmr/m/it/10 LNil$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto Overfull \hbox (2.5006pt too wide) in paragraph at lines 2874--2887 \OT1/cmr/m/it/10 4 3 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 split simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv LCons[]lprefix[]conv dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mo no-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.96495pt too wide) in paragraph at lines 2915--2919 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 ob-tain \OT1/cm r/m/it/10 x xs \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 LCons x xs $\OMS/cmsy/m/ n/10 2$ \OT1/cmr/m/it/10 Y \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv$\OT1 /cmr/m/n/10 )$[] Overfull \hbox (3.45793pt too wide) in paragraph at lines 2922--2924 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force dest$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF cha in$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 LCons[]lprefix[]conv lprefix[]LCons[]conv [37] Overfull \hbox (11.3537pt too wide) in paragraph at lines 3014--3036 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term llist$\OML/c mm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @ $$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 fixp[]rule[]uc$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$ \OT1/cmr/m/it/10 thm llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]strong[]in duct[]uc$\OMS/cmsy/m/n/10 g$ Overfull \hbox (10.92476pt too wide) in paragraph at lines 3050--3058 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [38] Overfull \hbox (10.92476pt too wide) in paragraph at lines 3225--3233 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [39] Overfull \hbox (11.56499pt too wide) in paragraph at lines 3404--3406 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst lhd[]lSu p$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 dest$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ] $ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 the[]equality$ \OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ [40] [41] [42] [43] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3719. [44] Overfull \hbox (16.78535pt too wide) in paragraph at lines 3905--3907 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs$ [] $ rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 rev[]induct$\OT1/cmr/m/n/10 )$$($\OT1/ cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Nil lappend[]llis t[]of[]llist[]of$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ] $ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4030. [45] [46] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4287. Overfull \hbox (15.20331pt too wide) in paragraph at lines 4386--4399 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 epred[]iadd1 [47] [48] Overfull \hbox (10.92476pt too wide) in paragraph at lines 4665--4673 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (18.88669pt too wide) in paragraph at lines 4677--4679 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 subst $\OT1/cmr/m /n/10 ($\OT1/cmr/m/it/10 1 2 3$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lfp$\OML/cmm /m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (17.23381pt too wide) in paragraph at lines 4692--4705 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/ 10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Overfull \hbox (19.53375pt too wide) in paragraph at lines 4711--4728 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lfp$\OML/cmm/m/ it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF llength[]mono llength[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it /10 fold bot[]enat[]def$\OML/cmm/m/it/10 ;$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 4728. [49] Overfull \hbox (17.11995pt too wide) in paragraph at lines 4940--4953 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\ OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff [50] [51] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5331--5339 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [52] [53] [54] Overfull \hbox (10.92476pt too wide) in paragraph at lines 5786--5794 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [55] [56] [57] [58] Overfull \hbox (25.67209pt too wide) in paragraph at lines 6689--6693 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 LCons \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases m rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/1 0 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 )$$($\OT1/cm r/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]Suc[]right$\O T1/cmr/m/n/10 )$[] [59] Overfull \hbox (68.23685pt too wide) in paragraph at lines 6786--6790 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Cons \OT1/cmr/bx/n/10 thus \OT1/cm r/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases n$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr /m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (27.84201pt too wide) in paragraph at lines 6882--6895 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldrop[]LCons iadd[]Suc[]righ t split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it /10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.39761pt too wide) in paragraph at lines 6900--6917 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct xs ar-bi-trar y$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 n m$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltake[]LCons ldrop[]LCons sp lit$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 6917. [60] [61] [62] Overfull \hbox (1.621pt too wide) in paragraph at lines 7327--7330 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/c mr/m/n/10 ($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ex I$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 = $\OT1/cmr/m/it/10 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/1 0 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmet ric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (19.0108pt too wide) in paragraph at lines 7336--7338 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 in-tr o$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 wh ere \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc n \OT1/cmr/bx/n/1 0 for \OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ileI1 simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] [63] Overfull \hbox (28.40157pt too wide) in paragraph at lines 7638--7651 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis eSuc[]enat eSu c[]plus[]1 ltake[]plus[]conv[]lappend ldrop[]enat ldropn[]Suc[]conv[]ldropn [64] [65] [66] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sqsubseteq' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8032. [67] Overfull \hbox (5.19078pt too wide) in paragraph at lines 8236--8249 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def lnull[]d ef neq[]LNil[]conv [68] [69] Overfull \hbox (4.94086pt too wide) in paragraph at lines 8503--8516 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 prefix[]def lprefix[]conv[]lappend$\OT1/cmr/m/n/1 0 )$$($\OT1/cmr/m/it/10 metis lfinite[]lappend lfinite[]llist[]of Overfull \hbox (21.38031pt too wide) in paragraph at lines 8611--8616 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lSup A$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 enat n \OT1/c mr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 lfinite[]conv[]llength[]enat Overfull \hbox (2.40771pt too wide) in paragraph at lines 8620--8623 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 fi-nite $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 llength ` A$\OT1/cmr/m/n/10 )$ \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ( $\OT1/cmr/m/it/10 rule finite[]subset$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 sim p add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 finite[]lessThan[]enat[]iff$\OT1/cmr/ m/n/10 )$[] [70] Overfull \hbox (13.92545pt too wide) in paragraph at lines 8799--8812 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llcp[]eq[]0[]iff epred[]llcp [71] Overfull \hbox (10.21999pt too wide) in paragraph at lines 8818--8831 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 iadd[]is[]0 llcp[]eq[]0[]iff Overfull \hbox (14.39069pt too wide) in paragraph at lines 8836--8849 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis add[]0[]right lappend[]LNil2 llcp[]LNil1 llcp[]lappend[]same lprefix[]conv[]lappend$\OT1/cmr /m/n/10 )$[] Overfull \hbox (52.74213pt too wide) in paragraph at lines 8897--8899 \OT1/cmr/m/it/10 exI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 x$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 Suc 0$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/ cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 iadd[]Suc[]right zero []enat[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[ ] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 8966. [72] Overfull \hbox (5.10889pt too wide) in paragraph at lines 9073--9086 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1 /cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff Overfull \hbox (14.78528pt too wide) in paragraph at lines 9140--9148 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac [73] Overfull \hbox (2.44716pt too wide) in paragraph at lines 9295--9298 [][] \OT1/cmr/bx/n/10 thus \OT1/cmr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr /m/n/10 ($\OT1/cmr/m/it/10 cases ys n rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 case[]product co$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 enat$\OML/cmm/m/it/1 0 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr/m/it/10 simp[]all[] [74] [75] [76] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9748--9761 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9767--9780 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.11893pt too wide) in paragraph at lines 9788--9805 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat[]min[]eq[]0[]iff lt l[]ltake epred[]llength$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 9805. [77] Overfull \hbox (10.92476pt too wide) in paragraph at lines 9859--9867 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ \OT1/cmr/m /it/10 PROP ?mono \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr /bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \O T1/cmr/m/it/10 Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (0.88739pt too wide) in paragraph at lines 9893--9906 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mono1$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cmr /m/it/10 simp[] Overfull \hbox (3.18733pt too wide) in paragraph at lines 9912--9925 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule llist$\OML/cmm/ m/it/10 :$\OT1/cmr/m/it/10 fixp[]preserves[]mcont1$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF ltakeWhile[]mono ltakeWhile[]conv[]fixp$\OT1/cmr/m/n/10 ]$$)$ \OT1/cm r/m/it/10 simp[] [78] [79] Overfull \hbox (5.86385pt too wide) in paragraph at lines 10306--10308 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 llength[]ltakeWhile[]lt[]iff$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 llength $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 ltake While P xs$\OT1/cmr/m/n/10 )$ $\OML/cmm/m/it/10 <$ \OT1/cmr/m/it/10 llength xs $\OMS/cmsy/m/n/10 []!$ $\OT1/cmr/m/n/10 ($$\OMS/cmsy/m/n/10 9 $\OT1/cmr/m/it/1 0 x$\OMS/cmsy/m/n/10 2$\OT1/cmr/m/it/10 lset Overfull \hbox (23.46579pt too wide) in paragraph at lines 10431--10444 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 no t[]lnull[]conv [80] [81] Overfull \hbox (4.60457pt too wide) in paragraph at lines 10598--10606 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 llength[]ltakeWhile[]all$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 llen gth[]eq[]infty[]conv[]lfinite$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1 /cmr/m/n/10 ]$[] Overfull \hbox (34.96571pt too wide) in paragraph at lines 10694--10707 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m/n /10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [82] Overfull \hbox (6.35873pt too wide) in paragraph at lines 10905--10918 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]eq[]infty[]conv[]l finite lfinite[]ltakeWhile$\OT1/cmr/m/n/10 )$[] Overfull \hbox (43.52377pt too wide) in paragraph at lines 10925--10938 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 ldropWhile[]eq[]ldrop llength[]ldrop llength[]lta keWhile[]all ltakeWhile[]all[]conv [83] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 10961. [84] Overfull \hbox (31.74066pt too wide) in paragraph at lines 11315--11317 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 dest$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 step llist[]all2[]llengthD [85] Overfull \hbox (25.92279pt too wide) in paragraph at lines 11331--11333 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases lnull xs $\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 step simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/cm r/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lnth[ ]0[]conv[]lhd$\OT1/cmr/m/n/10 )$[] [86] Overfull \hbox (37.6261pt too wide) in paragraph at lines 11639--11644 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth ys n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 ltake $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llength xs$\OT 1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 n \OT1/ cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lnth[]ltake$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$[] Overfull \hbox (4.15424pt too wide) in paragraph at lines 11644--11649 [][] \OT1/cmr/bx/n/10 also from \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 have \OT 1/cmr/m/it/10 lnth $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 lappend xs xs$ [] $$\OT1 /cmr/m/n/10 )$ \OT1/cmr/m/it/10 n $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lnth xs n \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 lnth[]lappend1$\OT1/cmr/m/n/10 )$[] [87] Overfull \hbox (15.4463pt too wide) in paragraph at lines 11688--11690 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 neq[]LNil[]conv lnul l[]def LNil[]eq[]lmap Overfull \hbox (24.38661pt too wide) in paragraph at lines 11696--11698 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr /m/it/10 auto dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lnullD llis t[]all2[]lhdD llist[]all2[]ltlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (7.40894pt too wide) in paragraph at lines 11742--11749 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 enat[]coinduct$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$ \OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv [88] Overfull \hbox (12.14566pt too wide) in paragraph at lines 11911--11913 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 image[]image dest$\OT1/cmr/m/n/10 :$ \ OT1/cmr/m/it/10 Y llist[]all2[]lnullD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 rev[]image[]eqI$\OT1/cmr/m/n/10 )$$+$[] [89] Overfull \hbox (38.50298pt too wide) in paragraph at lines 11980--11981 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12063. [90] Overfull \hbox (18.37143pt too wide) in paragraph at lines 12252--12256 [][] \OT1/cmr/bx/n/10 case \OT1/cmr/m/it/10 Suc \OT1/cmr/bx/n/10 thus \OT1/c mr/m/it/10 ?case \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases x s$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$ \OT1/cmr/m/it/10 llast[]LCons$\OT1/cmr/m/n/10 )$[] [91] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12334. [92] Overfull \hbox (5.61943pt too wide) in paragraph at lines 12468--12472 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/c mr/m/it/10 chain[]lprefix[]ltl chain in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldistinct[]ltlI Overfull \hbox (17.75882pt too wide) in paragraph at lines 12506--12508 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 ldistinct[]lSup chain[]imageI mcont[ ]monoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [93] [94] Overfull \hbox (0.21182pt too wide) in paragraph at lines 12872--12889 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 not[]lnull[]conv des t$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lset[]lzipD2$\OT1/cmr/m/n/10 )$ Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 12889. [95] Overfull \hbox (3.13603pt too wide) in paragraph at lines 13020--13025 [][] \OT1/cmr/bx/n/10 more-over have \OT1/cmr/m/it/10 ?ltl \OT1/cmr/bx/n/10 us -ing \OT1/cmr/m/it/10 chain sorted \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]ltl lsorted[]ltlI$\OT1/cmr/m/n/10 )$[] [96] Overfull \hbox (11.49773pt too wide) in paragraph at lines 13106--13108 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 mcont[]contD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF mcont$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 lsorted[]lSup chain[]imageI mcont[]m onoD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (12.42061pt too wide) in paragraph at lines 13121--13134 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML/cmm/m /it/10 :$\OT1/cmr/m/it/10 admissibleI$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 aut o dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lsorted[]lprefixD$\OT1/cmr/m/n/10 [$ \OT1/cmr/m/it/10 rotated$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 chain[]lprefix[]lSup$\OT1/cmr/m/n/10 )$[] Overfull \hbox (4.57834pt too wide) in paragraph at lines 13157--13170 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct n ar-bi-trary $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 f astforce simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ldropn[]Suc lsorted[]LCon s$ [] $ ldropn[]lnull [97] Overfull \hbox (1.39157pt too wide) in paragraph at lines 13303--13310 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lsorted[]coinduct$ [] $$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mon o-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [98] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 13397. [99] [100] [101] [102] [103] [104] [105] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 14351. [106] Overfull \hbox (5.09007pt too wide) in paragraph at lines 14626--14639 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 drule eq[]LConsD$\OT 1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m /it/10 exI simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ltl[]lfilter o[]def ldr opWhile[]eq[]LNil[]iff [107] [108] [109] [110] Overfull \hbox (14.26587pt too wide) in paragraph at lines 15252--15254 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fastforce simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]snocL1[]conv[]LCons2$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 symmetric$\OML/cmm/m/it/10 ;$ \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 =$\OT1/cmr/m/it/10 lappend [111] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15420--15421 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [112] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 15579. [113] [114] [115] Overfull \hbox (38.50298pt too wide) in paragraph at lines 15952--15953 [][] \OT1/cmr/m/it/10 parallel[]fixp[]induct[]1[]1$\OT1/cmr/m/n/10 [$\OT1/cmr/ m/it/10 OF llist[]partial[]function[]definitions llist[]partial[]function[]defi nitions [116] [117] Overfull \hbox (13.61642pt too wide) in paragraph at lines 16286--16290 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 concat[]xss$ [] $ nth[]n \OT 1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 xss \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lnth[]lappe nd2 lappend[]lnull1$\OT1/cmr/m/n/10 )$[] [118] Overfull \hbox (1.33876pt too wide) in paragraph at lines 16330--16332 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/ cmr/m/n/10 ($\OT1/cmr/m/it/10 1 2$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 atLeast0L essThan$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$)$$($\O T1/cmr/m/it/10 subst sum[]add[]nat[]ivl$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 si mp[]all$\OT1/cmr/m/n/10 )$[] [119] [120] Overfull \hbox (4.77174pt too wide) in paragraph at lines 16574--16576 [][] \OT1/cmr/bx/n/10 from \OT1/cmr/m/it/10 lfilter[]eq[]LConsD$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF []LCons x xs $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 lfi l-ter $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 xs$\OML/cmm/m/i t/10 :$ $\OMS/cmsy/m/n/10 :$ \OT1/cmr/m/it/10 lnull xs$\OT1/cmr/m/n/10 )$ \OT1/ cmr/m/it/10 xss[]$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$$]$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 16733. [121] [122] [123] [124] [125] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17381. Overfull \hbox (1.91145pt too wide) in paragraph at lines 17457--17459 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 lsum[]list[]LCons $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 lfi-nite xs $\OT 1/cmr/m/n/10 =[]\OMS/cmsy/m/n/10 )$ \OT1/cmr/m/it/10 lsum[]list $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 LCons x xs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 x $\OT1 /cmr/m/n/10 +$ \OT1/cmr/m/it/10 lsum[]list Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 17521. [126] [127] [128] [129] Overfull \hbox (11.00165pt too wide) in paragraph at lines 18136--18149 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set1[]pre[]llist[]def rel[]set[]def Overfull \hbox (11.00165pt too wide) in paragraph at lines 18155--18168 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]llist[]def vimage2p[]def rel[]fun[]def set2[]pre[]llist[]def rel[]set[]def [130] [131] [132]) (./Coinductive_List_Prefix.tex [133] [134] Overfull \hbox (17.24495pt too wide) in paragraph at lines 330--336 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 Sup[]llist[]def less[]eq[]llist[]def$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 abs[]def$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]upper llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 lub[]least$\OT1/cmr/m/n/10 )$[] ) (./Coinductive_Stream.tex [135] [136] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 243. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 395. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 395. [137] [138] [139] [140] Overfull \hbox (1.53853pt too wide) in paragraph at lines 1044--1057 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]stream[]def cr[]stream[]def in-tro$\OT1/ cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 rel[]funI rel-comppI rel[]setI [141] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\Rightarrow' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 1281. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 1281. [142] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1466. [143] Overfull \hbox (6.55463pt too wide) in paragraph at lines 1618--1624 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 bot[]enat[]def in-tro$\OT1/cmr/m/n/10 !$$:$ \OT1/cmr/m/it/10 admiss ible[]all admissible[]imp admissible[]eq[]mcontI Overfull \hbox (32.81557pt too wide) in paragraph at lines 1702--1707 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 step \OT1/cmr/bx/n/10 un-fol d-ing \OT1/cmr/m/it/10 eq \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/ 10 auto simp$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 scount[]simps card[]image zero []notin[]Suc[]image [144] Overfull \hbox (1.49925pt too wide) in paragraph at lines 1952--1954 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it /10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 sfirst$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 simps$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 of P $\OML/cmm/m/it/10 ! $$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm$\OT1/cmr/m/n/10 )$[] [145] Overfull \hbox (2.3468pt too wide) in paragraph at lines 2024--2027 [][] \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/10 sdrop$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 simps $\OMS/cmsy/m/n/10 ^^C$ \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 cases P $\OML/cmm/m/it/10 !$$\OT1/cmr/m/n/10 )$ $($\OT1/ cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ $\OMS/cmsy/m/n/10 ^^C$$^^C$ \OT1/c mr/m/it/10 eSuc[]enat$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n /10 ]$$)$[] [146] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2121. Overfull \hbox (28.19022pt too wide) in paragraph at lines 2129--2142 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 stakeWhile[]def LCons[]llist[]of[]stream$\OT1/cmr/m/n/ 10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 LCons[]llist[]of[]stream$\OT1/cmr/m/n/10 )$[] ) (./TLList.tex [147] [148] [149] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 465. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 465. [150] [151] [152] [153] Overfull \hbox (3.70673pt too wide) in paragraph at lines 1175--1188 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 4 simp add$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 pcr[]tllist[]def cr[]tllist[]def dest$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD in-tro$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 rel[]setI$\OT1/cmr/m/n/10 )$[] [154] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1377. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1421. [155] Overfull \hbox (23.40169pt too wide) in paragraph at lines 1470--1483 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 force simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 cr[]tllist[]def pcr[]tllist[]def terminal[]tllis t[]of[]llist dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]lfiniteD$\OT 1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1505. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1547. [156] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1702. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1799. [157] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 1948. [158] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2033. Overfull \hbox (21.524pt too wide) in paragraph at lines 2113--2115 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 tllist[]all2[]coinduct $\OT1/cmr/m/ n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]n ames tllist[]all2$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion tllist[ ]all2 [159] [160] Overfull \hbox (49.14331pt too wide) in paragraph at lines 2439--2452 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 trans-fer$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llist[]all2[]conv[ ]all[]lnth split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat [161] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2612. [162] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2729. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2826. [163] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 2930. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 3097. [164] Overfull \hbox (17.64603pt too wide) in paragraph at lines 3177--3190 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set1[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3196--3209 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set2[]pre[]tllist[]def rel[]set[]def Overfull \hbox (17.64603pt too wide) in paragraph at lines 3215--3228 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]pre[]tllist[]def vimage2p[]def rel[]fun[]def set3[]pre[]tllist[]def rel[]set[]def [165] Overfull \hbox (22.69978pt too wide) in paragraph at lines 3313--3315 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 tllist[]all2 C B $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 unfold[]tllist IS[]TNIL1 TER-MI-NAL1 THD1 TTL1 x$\OT1/cmr/m/ n/10 )$ $($\OT1/cmr/m/it/10 unfold[]tllist Overfull \hbox (8.84482pt too wide) in paragraph at lines 3414--3427 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 rel[]fun[]def tllist[]all2[]tmap1 tllist[]all2[]t map2 elim$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]mono$\OT1/cmr/m/n/1 0 )$[] [166] [167] Overfull \hbox (6.9575pt too wide) in paragraph at lines 3655--3657 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases $\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]T Cons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 Overfull \hbox (4.40196pt too wide) in paragraph at lines 3672--3674 [][] \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 cases$\OT1/cmr/m/n/10 ($\OT1/cmr /m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]TC ons1 tllist[]all2[]TCons2 tllist[]all2[]TNil1 ) (./Quotient_Coinductive_List.tex [168] Overfull \hbox (13.30737pt too wide) in paragraph at lines 168--181 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]llist[]all2 symp []llist[]all2 transp[]llist[]all2$\OT1/cmr/m/n/10 )$[] [169] Overfull \hbox (52.5827pt too wide) in paragraph at lines 202--204 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 a$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1 /cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotie nt3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [170] Overfull \hbox (4.68169pt too wide) in paragraph at lines 339--352 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient[]lmap[]Abs[]Rep Quotient[]llist[]all2[]lmap[]Rep Overfull \hbox (2.09499pt too wide) in paragraph at lines 433--446 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 fact lmap[]transfer$ \OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it /10 llist[]all2[]conv[]all[]lnth lmap[]eq[]lmap[]conv[]llist[]all2 [171] Overfull \hbox (73.35773pt too wide) in paragraph at lines 515--516 [][] $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\ OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/c mr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient[]lmap[]Abs[]Rep$\ OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Quotient_TLList.tex [172] Overfull \hbox (1.53548pt too wide) in paragraph at lines 79--80 [][] \OT1/cmr/bx/n/10 shows $\OT1/cmr/m/n/10 ($$($\OT1/cmr/m/it/10 id $\OMS/cm sy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep$\OT1/cmr/m/n/ 10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cm r/m/it/10 Rep$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it /10 >$ \OT1/cmr/m/it/10 id $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Abs$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 case[]sum [173] Overfull \hbox (23.27394pt too wide) in paragraph at lines 254--267 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 equivp[]reflp[]symp[]transp reflp[]tllist[]all2 sym p[]tllist[]all2 transp[]tllist[]all2$\OT1/cmr/m/n/10 )$[] Overfull \hbox (55.70293pt too wide) in paragraph at lines 327--340 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ts$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/1 0 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Quotient3[]rep[]reflp$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotien t3[]rep[]reflp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [174] Overfull \hbox (28.84264pt too wide) in paragraph at lines 429--442 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 blast in-tro$\OT1/cm r/m/n/10 :$ \OT1/cmr/m/it/10 Quo-tient3I dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/ 10 Quotient3[]tmap[]Abs[]Rep Quotient3[]tllist[]all2[]tmap[]tmapI Overfull \hbox (3.84383pt too wide) in paragraph at lines 452--453 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 Quo-tient $\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 tllist[]all2 R1 R2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Abs 1 Abs2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tmap Rep1 Rep2$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 tllist[]all2 [175] Overfull \hbox (32.54527pt too wide) in paragraph at lines 511--513 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto 4 3 simp ad d$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]conv[]all[]tnth dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 lfinite[]llength[]enat not[]lfinite[]llength$\OT1 /cmr/m/n/10 )$[] [176] Overfull \hbox (8.50388pt too wide) in paragraph at lines 618--620 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto dest$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]is[]TNilD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]all2[]tfinite1[]terminalD tllist[]all2[]thdD Overfull \hbox (49.95847pt too wide) in paragraph at lines 657--665 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/cmr /m/n/10 :$ \OT1/cmr/m/it/10 fun[]eq[]iff map[]fun[]def comp[]def Quotient3[]rel []rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it /10 Quotient3[]rel[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (4.31384pt too wide) in paragraph at lines 679--680 \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Abs1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$^^@$$\OML/c mm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 ^^@$$^ ^@$$^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 Rep1 $\OMS/cmsy/m/n/10 ^^@$$^^@$$ ^^@$$\OML/cmm/m/it/10 >$ \OT1/cmr/m/it/10 tmap Abs3 Abs2$\OT1/cmr/m/n/10 )$ \OT 1/cmr/m/it/10 corec[]tllist $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 corec[]tllist[ ] Overfull \hbox (52.91345pt too wide) in paragraph at lines 693--695 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-b i-trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 b rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/ m/it/10 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 coinduct[]strong$\OT1/cmr/m /n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Q uotient3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (10.2469pt too wide) in paragraph at lines 693--695 \OT1/cmr/m/it/10 q1$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quotient3[]abs[]rep$\OT 1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q2$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 Quoti ent3[]abs[]rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF q3$\OT1/cmr/m/n/10 ]$ \OT1 /cmr/m/it/10 Quotient3[]tmap[]Abs[]Rep$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF ) (./Coinductive.tex [177]) (./Lazy_LList.tex Overfull \hbox (1.13655pt too wide) in paragraph at lines 60--61 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [178] [179] [180] [181] [182] [183]) (./Lazy_TLList.tex [184] Overfull \hbox (1.13655pt too wide) in paragraph at lines 61--62 [][] \OT1/cmr/m/it/10 partial[]term[]of ty-tok $\OT1/cmr/m/n/10 ($\OT1/cmr/m/i t/10 Quickcheck[]Narrowing$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Narrowing[]const ructor 1 $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 head$\OML/cmm/m/it/10 ;$ \OT1/cmr/ m/it/10 tail$\OT1/cmr/m/n/10 ]$$)$ [185] [186] [187] [188]) (./CCPO_Topology.tex [189] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\mskip' on input line 191. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `math shift' on input line 191. [190] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 348. [191] [192] Overfull \hbox (9.69476pt too wide) in paragraph at lines 733--737 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] [193] Overfull \hbox (9.69476pt too wide) in paragraph at lines 758--762 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 ev \OT1/cmr/bx/n/10 have \OT1/cm r/m/it/10 even-tu-ally $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/1 0 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 False$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it /10 F \OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 eventually[]elim $\OT1/cmr/m/n/10 ($ \OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 order[]trans$\ OT1/cmr/m/n/10 )$[] Overfull \hbox (10.55899pt too wide) in paragraph at lines 817--819 [][] \OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 intro chain[]im ageI$\OT1/cmr/m/n/10 [$\OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 le[]a$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 op $\OMS/cmsy/m/n/10 ^^T$$\OT1/cmr/m/n/10 ]$ \OT1/cmr/ m/it/10 C$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \O T1/cmr/m/it/10 mcont[]def monotone[]def$\OT1/cmr/m/n/10 )$[] Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 835. [194] [195]) (./LList_CCPO_Topology.tex) (./TLList_CCPO.tex [196] [197] Overfull \hbox (10.85344pt too wide) in paragraph at lines 381--394 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq split$\OT1/cmr/m/n /10 :$ \OT1/cmr/m/it/10 if[]split[]asm dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Overfull \hbox (6.05344pt too wide) in paragraph at lines 401--414 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chainI$\OT1/cmr /m/n/10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[]ord[]def dest$\O T1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chainD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF assms$\OT1/cmr/m/n/10 ]$$)$[] [198] Overfull \hbox (17.85112pt too wide) in paragraph at lines 518--520 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def terminal[]tllist[]of[]llist image[]ima ge$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 :$ \OT1/cm r/m/it/10 rev[]image[]eqI Overfull \hbox (24.56375pt too wide) in paragraph at lines 523--525 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]upper$\OT1/cmr/m/n/10 [$\OT1/cmr/m/i t/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/ cmr/m/it/10 blast Overfull \hbox (25.60872pt too wide) in paragraph at lines 536--538 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule contrapos []np$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto in-tro$\OT1/cmr/m/n/10 !$$:$ \O T1/cmr/m/it/10 lprefix[]antisym chain[]lSup[]lprefix chain[]lprefix[]lSup Overfull \hbox (7.71898pt too wide) in paragraph at lines 536--538 \OT1/cmr/m/it/10 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tSup[]def image[] image A chain[]tllist[]llist[]of[]tllist$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 rep[]eq Overfull \hbox (59.82928pt too wide) in paragraph at lines 553--555 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image chain[]lprefix[]lSup chain[]tllist[]llist[]of[]t llist [199] Overfull \hbox (83.78731pt too wide) in paragraph at lines 561--565 \OT1/cmr/m/it/10 chain[]lprefix[]lSup chain[]tllist[]llist[]of[]tllist not[]lfi nite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN iffD1$\OT1/cmr/ m/n/10 ]$ \OT1/cmr/m/it/10 terminal[]tllist[]of[]llist Overfull \hbox (20.74199pt too wide) in paragraph at lines 607--609 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq tSup[]def image[]image not[]lfinite[]lprefix[]conv[]eq$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN Overfull \hbox (11.60599pt too wide) in paragraph at lines 628--632 [][] \OT1/cmr/bx/n/10 with \OT1/cmr/m/it/10 pre-fix \OT1/cmr/bx/n/10 have \OT1/cmr/m/it/10 lSup $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 llist[]of[]tllist ` A $\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 llist[]of[]tllist xs \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule lprefix[]antisym$\OT1/cmr/m/n/10 )$[ ] Overfull \hbox (24.05267pt too wide) in paragraph at lines 635--637 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule ccpo$\O ML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/cmr/m/n/10 [$\OT1/cmr/m /it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo$\OT1/cmr/m /n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT 1/cmr/m/it/10 auto Overfull \hbox (10.06415pt too wide) in paragraph at lines 635--637 \OT1/cmr/m/it/10 in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 chain[]tllist[]term inal$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF chain$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/ it/10 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lub simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 rep[]eq flat[] ord[]def$\OT1/cmr/m/n/10 )$[] [200] Overfull \hbox (10.475pt too wide) in paragraph at lines 665--667 [][] \OT1/cmr/bx/n/10 by $\OMS/cmsy/m/n/10 ^^@$$\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 rule ccpo$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 ccpo[]Sup[]least$\OT1/ cmr/m/n/10 [$\OT1/cmr/m/it/10 OF Partial[]Function$\OML/cmm/m/it/10 :$\OT1/cmr/ m/it/10 ccpo$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF flat[]interpretation$\OT1/cm r/m/n/10 ]$$]$$\OML/cmm/m/it/10 ;$ Overfull \hbox (0.63309pt too wide) in paragraph at lines 692--705 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s Overfull \hbox (0.63309pt too wide) in paragraph at lines 710--723 [][]\OT1/cmr/bx/n/10 by \OT1/cmr/m/it/10 unfold[]locales$\OT1/cmr/m/n/10 ($\OT1 /cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mk[]less[]def in -tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]antisym tllist[]ord[]tran s [201] [202] [203] [204] Overfull \hbox (19.03722pt too wide) in paragraph at lines 1257--1260 [][] \OT1/cmr/bx/n/10 us-ing \OT1/cmr/m/it/10 chain \OT1/cmr/bx/n/10 by$ \OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule chain[]imageI$\OT1/cmr/m/n/10 [$\OT1/cm r/m/it/10 OF chain[]subset$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp a dd$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 tllist[]ord[]ttlI$\OT1/cmr/m/n/10 )$[] Overfull \hbox (18.68668pt too wide) in paragraph at lines 1342--1344 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mono2mono[]TCons$\OT1/cmr/m/n/10 [ $\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 monotone[ ]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 mono2mono$\OT1/cmr/m/n/10 ]$[] Overfull \hbox (11.84834pt too wide) in paragraph at lines 1371--1373 [][]\OT1/cmr/bx/n/10 lemmas \OT1/cmr/m/it/10 mcont2mcont[]TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 cont[]intro$\OT1/cmr/m/n/10 ]$ $=$ \OT1/cmr/m/it/10 mcont[] TCons$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 THEN tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 mcont2mcont$\OT1/cmr/m/n/10 ]$[] [205] Overfull \hbox (4.28688pt too wide) in paragraph at lines 1531--1548 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule mono-toneI$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto split$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/1 0 tl-list$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 split dest$\OT1/cmr/m/n/10 :$ \OT 1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF tnil$\OT1/cmr/m/ n/10 ]$ \OT1/cmr/m/it/10 mono-toneD$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF [206] Overfull \hbox (71.64563pt too wide) in paragraph at lines 1565--1583 [][] $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 term tl-list$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body b$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n/ 10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/c mr/m/it/10 fixp[]rule[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where b$\OT1/cmr/m /n/10 =$\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 ]$$\OMS/cmsy/m/n/10 g$ $\OT1/cmr/m/n /10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 thm tl-list$\OML/cmm/m/it/10 :$\OT1/ cmr/m/it/10 fixp[]induct[]uc$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 where ) (./TLList_CCPO_Examples.tex [207] [208]) (./Koenigslemma.tex [209] Overfull \hbox (1.35538pt too wide) in paragraph at lines 45--46 [][]\OT1/cmr/bx/n/10 where $[]$ \OT1/cmr/m/it/10 LCons n xs $\OMS/cmsy/m/n/10 2 $ \OT1/cmr/m/it/10 paths graph$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 n$ [] $ $\OM S/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 lset xs$\OT1/cmr/m/n/10 ;$ \OT1/cmr/m/it/10 l set xs $\OMS/cmsy/m/n/10 ^^R$ \OT1/cmr/m/it/10 ns $[]$ $\OT1/cmr/m/n/10 =[]\OMS /cmsy/m/n/10 )$ \OT1/cmr/m/it/10 n$ [] $ $\OMS/cmsy/m/n/10 2$ \OT1/cmr/m/it/10 reachable[]via [210] Overfull \hbox (64.58913pt too wide) in paragraph at lines 233--235 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp add$\OT1/ cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]assoc$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 metis lappend[]assoc lappend[]llist[]of[]LCons lappend[]llist[]of[]llist[] of [211] [212] [213] [214]) (./LMirror.tex [215] [216] Overfull \hbox (46.50336pt too wide) in paragraph at lines 194--196 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induction ar-bi- trary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it /10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[]code$\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$[$\OT1/cmr/m/it/10 symmetric$\OT1/ cmr/m/n/10 ]$ \OT1/cmr/m/it/10 del$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lappend[ ]code$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 2$\OT1/cmr/m/n/10 )$$)$[] Overfull \hbox (18.66428pt too wide) in paragraph at lines 241--248 [][]\OT1/cmr/bx/n/10 by $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 metis $\OT1/cmr/m/n /10 ($\OT1/cmr/m/it/10 hide[]lams$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 no[]type s$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 add$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 c ommute epred[]llength iadd[]Suc[]right lhd[]LCons[]ltl [217] Overfull \hbox (17.3283pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 acc acc$ [] $ xs xs$ [] $$\OT1/cmr/m/n/ 10 )$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[ ]lmirror[]aux ltl[]lmirror[]aux Overfull \hbox (61.63919pt too wide) in paragraph at lines 480--493 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases k m n rule$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 enat$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhau st$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OML/cmm/m/it/10 :$\OT 1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 case[]product enat$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 exhaust$\OT1/cmr/m/n/10 ]$$]$$)$$($\OT1/cmr/m/ it/10 simp[]all Overfull \hbox (4.2604pt too wide) in paragraph at lines 525--528 [][] \OT1/cmr/bx/n/10 us-ing []\OT1/cmr/m/it/10 lfinite acc[] \OT1/cmr/bx/n/ 10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/ cmr/m/it/10 llength[]lmirror[]aux dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lfin ite[]llength[]enat$\OT1/cmr/m/n/10 )$[] [218]) (./Hamming_Stream.tex [219] [220] Overfull \hbox (14.78528pt too wide) in paragraph at lines 326--334 [][] \OT1/cmr/bx/n/10 show \OT1/cmr/m/it/10 mono$\OT1/cmr/m/n/10 :$ $[]$\OT1/c mr/m/it/10 xs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 ?mono xs \OT1/cmr/bx/n/10 un -fold-ing \OT1/cmr/m/it/10 F[]def \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cm r/m/it/10 tactic $\OMS/cmsy/m/n/10 h h$ \OT1/cmr/m/it/10 Partial[]Function$\OML /cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]tac Overfull \hbox (16.9785pt too wide) in paragraph at lines 343--345 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cm r/m/n/10 ($\OT1/cmr/m/it/10 1 3 4$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 llist$\OM L/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono[]body[]fixp$\OT1/cmr/m/n/10 [$\OT1/cmr/m/ it/10 OF mono$\OT1/cmr/m/n/10 ]$$)$$($\OT1/cmr/m/it/10 auto simp add$\OT1/cmr/m /n/10 :$ \OT1/cmr/m/it/10 F[]def lmerge[]simps Overfull \hbox (13.73233pt too wide) in paragraph at lines 357--359 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 monotone[]lmerge$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 mono-tone $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rel[]prod lpre- fix lpre-fix$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 lpre-fix $\OT1/cmr/m/n/10 ($\O T1/cmr/m/it/10 case[]prod lmerge$\OT1/cmr/m/n/10 )$[] Overfull \hbox (11.89853pt too wide) in paragraph at lines 367--369 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mono2 mono$\OT1/cmr/m/n/10 )$$+$[] Overfull \hbox (16.8158pt too wide) in paragraph at lines 427--429 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 erule conjE$\OMS/ cmsy/m/n/10 j$\OT1/cmr/m/it/10 rule allI conjI cont[]intro$\OMS/cmsy/m/n/10 j$\ OT1/cmr/m/it/10 simp$\OMS/cmsy/m/n/10 j$\OT1/cmr/m/it/10 erule allE$\OML/cmm/m/ it/10 ;$ \OT1/cmr/m/it/10 erule llist$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 mcont 2mcont$\OT1/cmr/m/n/10 )$$+$[] [221] [222] Overfull \hbox (13.33519pt too wide) in paragraph at lines 704--717 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 coinduction ar-bi-tr ary$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 xs ys$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/i t/10 auto 4 3 simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 lhd[]lmerge ltl[]lme rge not[]lnull[]conv [223] Overfull \hbox (51.39769pt too wide) in paragraph at lines 1000--1014 [][]\OT1/cmr/bx/n/10 unfolding \OT1/cmr/m/it/10 hamming[]def \OT1/cmr/bx/n/10 b y$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 induct rule$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/ it/10 ham-ming$ [] $$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 fixp[]induct$\OT1/cmr/ m/n/10 )$$($\OT1/cmr/m/it/10 auto 6 6 dest$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 in[]lset[]lmergeD$\OT1/cmr/m/n/10 )$[] Overfull \hbox (24.94225pt too wide) in paragraph at lines 1029--1034 [][] \OT1/cmr/bx/n/10 then ob-tain \OT1/cmr/m/it/10 n \OT1/cmr/bx/n/10 where \ OT1/cmr/m/it/10 n$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 llength ham-ming $\OT1/cm r/m/n/10 =$ \OT1/cmr/m/it/10 enat n \OT1/cmr/bx/n/10 un-fold-ing \OT1/cmr/m/it/ 10 lfinite[]conv[]llength[]enat [224] Overfull \hbox (10.80869pt too wide) in paragraph at lines 1055--1057 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst $\OT1/cmr/ m/n/10 ($\OT1/cmr/m/it/10 asm$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 hamming[]unfo ld$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 cases n$\OML/cmm/m/it/10 ;$ \OT1/cmr/m /it/10 auto simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 zero[]enat[]def$\OT1/c mr/m/n/10 [$\OT1/cmr/m/it/10 symmetric$\OT1/cmr/m/n/10 ]$ Overfull \hbox (39.67842pt too wide) in paragraph at lines 1087--1089 \OT1/cmr/m/it/10 in[]lset[]lmergeD in-tro$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 s mooth[]ge[]Suc0 lsorted[]lmerge lsorted[]lmap mono-toneI ldistinct[]lmerge [225] Overfull \hbox (12.65755pt too wide) in paragraph at lines 1208--1210 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 subst hammin g[]unfold$\OT1/cmr/m/n/10 )$$($\OT1/cmr/m/it/10 auto 4 4 simp add$\OT1/cmr/m/n/ 10 :$ \OT1/cmr/m/it/10 not[]less lsorted[]lmap lsorted[]lmerge ) (./Resumption.tex Overfull \hbox (10.0379pt too wide) in paragraph at lines 6--6 []\OT1/cmr/bx/n/14.4 Manual con-struc-tion of a re-sump-tion co-datatype [226] Overfull \hbox (4.26314pt too wide) in paragraph at lines 37--37 []\OT1/cmr/bx/n/12 Auxiliary def-i-ni-tions and lem-mata sim-i-lar to \OT1/cmr/ m/it/12 Old[]Datatype Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Package hyperref Warning: Token not allowed in a PDF string (PDFDocEncoding): (hyperref) removing `\sfcode' on input line 37. Overfull \hbox (7.62393pt too wide) in paragraph at lines 39--40 \OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Lim[]mono$\OT1/cmr/m/n/10 :$ $($$[]$\OT 1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 rs d $\OMS/cmsy/m/n/10 ^^R $ \OT1/cmr/m/it/10 rs$ [] $ d$\OT1/cmr/m/n/10 )$ $=[]\OMS/cmsy/m/n/10 )$ \OT1/c mr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs $\OMS/cmsy/ m/n/10 ^^R$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim Overfull \hbox (0.97466pt too wide) in paragraph at lines 75--77 []\OT1/cmr/m/n/10.95 Inverse for \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/i t/10.95 :$\OT1/cmr/m/it/10.95 Lim \OT1/cmr/m/n/10.95 like \OT1/cmr/m/it/10.95 O ld[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.95 Split \OT1/cmr/m/n/10.95 and \OT1/cmr/m/it/10.95 Old[]Datatype$\OML/cmm/m/it/10.95 :$\OT1/cmr/m/it/10.9 5 Case Overfull \hbox (16.13928pt too wide) in paragraph at lines 153--155 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 ntrunc[]Lim $\OT1/cmr/m/n/10 [$\OT1 /cmr/m/it/10 simp$\OT1/cmr/m/n/10 ]$$:$ \OT1/cmr/m/it/10 ntrunc $\OT1/cmr/m/n/1 0 ($\OT1/cmr/m/it/10 Suc k$\OT1/cmr/m/n/10 )$ $($\OT1/cmr/m/it/10 Old[]Datatype $\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim rs$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/i t/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 Lim [227] Overfull \hbox (27.08263pt too wide) in paragraph at lines 195--197 [][] \OT1/cmr/bx/n/10 where \OT1/cmr/m/it/10 BRANCH c rs $\OT1/cmr/m/n/10 =$ \O T1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 In1 $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Scons $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cm m/m/it/10 :$\OT1/cmr/m/it/10 Leaf $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Inl c$\OT 1/cmr/m/n/10 )$$)$ $($\OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cm r/m/it/10 Lim Overfull \hbox (39.99089pt too wide) in paragraph at lines 200--201 []\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 case[]RESUMPTION $\OT1/cmr/m/n/1 0 :$$:$ $($$ [] $\OT1/cmr/m/it/10 a $\OMS/cmsy/m/n/10 )$ $ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/ it/10 b $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$($$ [] $\OT1/cmr/m/it/10 c $\O T1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/ it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cm r/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree$\OT1/cmr/m/n/ 10 )$ Overfull \hbox (6.96573pt too wide) in paragraph at lines 236--237 [][] \OT1/cmr/bx/n/10 shows \OT1/cmr/m/it/10 case[]RESUMPTION[]TERMINAL$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION t l br $\OT1/cmr/m/n/10 ($\OT1/c mr/m/it/10 TERMINAL [228] Overfull \hbox (32.29482pt too wide) in paragraph at lines 239--247 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 case[]RESUMPTION[]def TERMINAL[]def LINEAR[]de f BRANCH[]def Overfull \hbox (11.58765pt too wide) in paragraph at lines 359--360 \OT1/cmr/bx/n/10 typedef $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\ OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 re-sump-tion $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 b $\OT1/cmr/m/n/10 +$ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cm r/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 dtree [229] Overfull \hbox (4.37408pt too wide) in paragraph at lines 391--393 [][]\OT1/cmr/bx/n/10 definition \OT1/cmr/m/it/10 Branch $\OT1/cmr/m/n/10 :$$:$ $ [] $\OT1/cmr/m/it/10 c $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr /m/it/10 d $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OM L/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it /10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m /it/10 re-sump-tion$\OT1/cmr/m/n/10 )$ $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($ $ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m /it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\ OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[] Overfull \hbox (6.82832pt too wide) in paragraph at lines 406--414 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto simp add$\OT 1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def simp add $\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (29.8056pt too wide) in paragraph at lines 429--430 [][] \OT1/cmr/bx/n/10 and \OT1/cmr/m/it/10 Rep[]resumption[]Linear$\OT1/cmr/m/ n/10 :$ \OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Li near b r$\OT1/cmr/m/n/10 )$ $=$ \OT1/cmr/m/it/10 LIN-EAR b $\OT1/cmr/m/n/10 ($\ OT1/cmr/m/it/10 Rep[]resumption Overfull \hbox (16.84444pt too wide) in paragraph at lines 454--455 [][] \OT1/cmr/m/it/10 case[]RESUMPTION t $\OT1/cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 b r$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 l b $\OT1/cmr/m/ n/10 ($\OT1/cmr/m/it/10 Abs[]resumption r$\OT1/cmr/m/n/10 )$$)$ $($$\OML/cmm/m/ it/10 ^^U$\OT1/cmr/m/it/10 c rs$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 br c $\OT1 /cmr/m/n/10 ($$\OML/cmm/m/it/10 ^^U$\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 :$ \OT1 /cmr/m/it/10 Abs[]resumption Overfull \hbox (61.77362pt too wide) in paragraph at lines 461--474 [][]\OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 simp[]all add$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[]def Branch[]def case[]resum ption[]def Abs[]resumption[]inverse [230] Overfull \hbox (41.57692pt too wide) in paragraph at lines 515--524 [][] \OT1/cmr/m/it/10 Nit-pick$\OML/cmm/m/it/10 :$\OT1/cmr/m/it/10 register[]c odatatype $\OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 typ $\OT1/cmr /m/n/10 ($$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$ \OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m /it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 re-sump-tion$\OMS/cmsy/m/n/10 g$ $ \OT1/cmr/m/n/10 @$$\OMS/cmsy/m/n/10 f$\OT1/cmr/m/it/10 const[]name case[]resump tion$\OMS/cmsy/m/n/10 g$[] [231] Overfull \hbox (4.62018pt too wide) in paragraph at lines 673--675 [][]\OT1/cmr/bx/n/10 primrec \OT1/cmr/m/it/10 RESUMPTION[]corec[]aux $\OT1/cmr/ m/n/10 :$$:$ \OT1/cmr/m/it/10 nat $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it/10 e $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/it /10 a$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 b$\OML/cmm/m/it/10 ;$$ [] $\OT1 /cmr/m/it/10 c$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 d$\OML/cmm/m/it/10 ;$$ [] $\OT1/cmr/m/it/10 e$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 resumption[]corec$\ OT1/cmr/m/n/10 )$ [232] Overfull \hbox (10.79494pt too wide) in paragraph at lines 719--721 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule conjI str ip LINEAR[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upper$\OT1/cmr/m/n/10 ]$ \OT1/cmr/m/it/10 BRANCH[]mono$\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 OF UN[]upp er$\OT1/cmr/m/n/10 ]$ Overfull \hbox (17.23096pt too wide) in paragraph at lines 814--816 [][]\OT1/cmr/bx/n/10 apply$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 auto split$\OT1/c mr/m/n/10 :$ \OT1/cmr/m/it/10 resumption[]corec$\OML/cmm/m/it/10 :$\OT1/cmr/m/i t/10 splits simp add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/it/10 Terminal[]def Linear[] def Branch[]def Overfull \hbox (5.21599pt too wide) in paragraph at lines 829--830 []\OT1/cmr/bx/n/10 coinductive \OT1/cmr/m/it/10 Eq[]RESUMPTION $\OT1/cmr/m/n/10 :$$:$ $($$ [] $\OT1/cmr/m/it/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\ OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ $ [] $\OT1/cmr/m/ it/10 d$\OT1/cmr/m/n/10 )$ \OT1/cmr/m/it/10 Old[]Datatype$\OML/cmm/m/it/10 :$\O T1/cmr/m/it/10 dtree $\OMS/cmsy/m/n/10 )$ $\OT1/cmr/m/n/10 ($$ [] $\OT1/cmr/m/i t/10 c$\OT1/cmr/m/n/10 +$$ [] $\OT1/cmr/m/it/10 b$\OT1/cmr/m/n/10 +$$ [] $\OT1/ cmr/m/it/10 a$\OML/cmm/m/it/10 ;$ [233] [234] Overfull \hbox (28.5241pt too wide) in paragraph at lines 995--998 [][] \OT1/cmr/bx/n/10 hence $[]$\OT1/cmr/m/it/10 k$\OML/cmm/m/it/10 :$ \OT1/cm r/m/it/10 ntrunc k r $\OT1/cmr/m/n/10 =$ \OT1/cmr/m/it/10 ntrunc k r$ [] $ \OT1 /cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 rule Eq[]RESUMPTION[]implies []ntrunc[]equality$\OT1/cmr/m/n/10 )$[] Overfull \hbox (38.82811pt too wide) in paragraph at lines 1028--1030 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 Eq[]RESUMPTION[]I $\OT1/cmr/m/n/10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]names Eq[]RESUMPTION$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion Overfull \hbox (14.31752pt too wide) in paragraph at lines 1062--1064 [][]\OT1/cmr/bx/n/10 lemma \OT1/cmr/m/it/10 resumption[]equalityI $\OT1/cmr/m/n /10 [$\OT1/cmr/m/it/10 consumes 1$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]na mes Eq[]resumption$\OML/cmm/m/it/10 ;$ \OT1/cmr/m/it/10 case[]conclusion [235] [236] Overfull \hbox (21.40091pt too wide) in paragraph at lines 1237--1239 [][] \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 cases r$\OT1 /cmr/m/n/10 )$$($\OT1/cmr/m/it/10 simp[]all add$\OT1/cmr/m/n/10 :$ \OT1/cmr/m/i t/10 h h$ [] $ Rep[]resumption[]constructors Eq[]RESUMPTION[]refl Overfull \hbox (89.4882pt too wide) in paragraph at lines 1284--1287 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 eq$\OT1/cmr/m/n/10 :$ $($$\OML/cm m/m/it/10 ^^U$\OT1/cmr/m/it/10 x$\OML/cmm/m/it/10 :$ \OT1/cmr/m/it/10 Rep[]resu mption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1/cmr/m/n/10 )$$)$ $=$ \OT1/c mr/m/it/10 RESUMPTION[]corec f \OT1/cmr/bx/n/10 by$\OT1/cmr/m/n/10 ($\OT1/cmr/m /it/10 rule equals[]RESUMPTION[]corec$\OT1/cmr/m/n/10 )$[] Overfull \hbox (29.55049pt too wide) in paragraph at lines 1287--1289 [][] \OT1/cmr/bx/n/10 hence \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 Rep[]resumption $\OT1/cmr/m/n/10 ($\OT1/cmr/m/it/10 h x$\OT1 /cmr/m/n/10 )$$)$ $=$ \OT1/cmr/m/it/10 Abs[]resumption $\OT1/cmr/m/n/10 ($\OT1/ cmr/m/it/10 RESUMPTION[]corec [237]) (./Coinductive_Examples.tex)) [238] (./root.aux) ) (see the transcript file for additional information) Output written on root.pdf (238 pages, 736872 bytes). Transcript written on root.log. *** exception THM 0 raised (line 328 of "drule.ML"): *** OF: no unifiers *** \closed ?s; \x. isCont ?f x\ *** \ closed (?f -` ?s) *** isCont (\x. (f x, g x)) ?a *** closed {(x, y). llist_all2 ?R x y} *** At command "using" (line 194 of "~~/afp/thys/Coinductive/Examples/LList_CCPO_Topology.thy")