| author | wenzelm |
| Fri, 03 Apr 2015 20:52:17 +0200 | |
| changeset 59920 | 86d302846b16 |
| parent 58889 | 5b7a9633cfa8 |
| child 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 {* Coinduction Method *} theory Coinduction imports Ctr_Sugar begin ML_file "Tools/coinduction.ML" end