author | wenzelm |
Thu, 30 Oct 2014 22:45:19 +0100 | |
changeset 58839 | ccda99401bc8 |
parent 58814 | 4c0ad4162cb7 |
child 58889 | 5b7a9633cfa8 |
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. *) header {* Coinduction Method *} theory Coinduction imports Ctr_Sugar begin ML_file "Tools/coinduction.ML" end