| author | nipkow | 
| Tue, 19 Jan 2016 11:46:54 +0100 | |
| changeset 62204 | 7f5579b12b0a | 
| parent 60758 | d8d85a8172b5 | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Coinduction.thy Author: Johannes Hölzl, TU Muenchen Author: Dmitriy Traytel, TU Muenchen Copyright 2013 Coinduction method that avoids some boilerplate compared to coinduct. *) section \<open>Coinduction Method\<close> theory Coinduction imports Ctr_Sugar begin ML_file "Tools/coinduction.ML" end