(* Title: HOL/Datatype_Examples/Milner_Tofte.thy Author: Dmitriy Traytel, ETH Zürich Copyright 2015 Modernized version of an old development by Jacob Frost Based upon the article Robin Milner and Mads Tofte, Co-induction in Relational Semantics, Theoretical Computer Science 87 (1991), pages 209-220. Written up as Jacob Frost, A Case Study of Co_induction in Isabelle/HOL Report 308, Computer Lab, University of Cambridge (1993). *) section ‹Milner-Tofte: Co-induction in Relational Semantics› theory Milner_Tofte imports Main begin typedecl Const typedecl ExVar typedecl TyConst