author | immler |
Thu, 09 Jun 2016 16:04:20 +0200 | |
changeset 63263 | c6c95d64607a |
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