(* Title: HOL/Corec_Examples/Tests/Merge_Poly.thy Author: Aymeric Bouzy, Ecole polytechnique Author: Jasmin Blanchette, Inria, LORIA, MPII Copyright 2015, 2016 Tests polymorphic merges. *) section ‹Tests Polymorphic Merges› theory Merge_Poly imports "HOL-Library.BNF_Corec" begin subsection ‹A Monomorphic Example› codatatype r = R (rhd: nat) (rtl: r)