| author | blanchet |
| Thu, 11 Sep 2014 19:45:42 +0200 | |
| changeset 58315 | 6d8458bc6e27 |
| parent 54555 | e8c5e95d338b |
| child 58814 | 4c0ad4162cb7 |
| 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" setup Coinduction.setup end