| author | wenzelm | 
| Thu, 20 Aug 2015 17:39:07 +0200 | |
| changeset 60986 | 077f663b6c24 | 
| parent 60758 | d8d85a8172b5 | 
| permissions | -rw-r--r-- | 
| 54540 | 1 | (* Title: HOL/Coinduction.thy | 
| 54026 | 2 | Author: Johannes Hölzl, TU Muenchen | 
| 3 | Author: Dmitriy Traytel, TU Muenchen | |
| 4 | Copyright 2013 | |
| 5 | ||
| 6 | Coinduction method that avoids some boilerplate compared to coinduct. | |
| 7 | *) | |
| 8 | ||
| 60758 | 9 | section \<open>Coinduction Method\<close> | 
| 54026 | 10 | |
| 11 | theory Coinduction | |
| 54555 | 12 | imports Ctr_Sugar | 
| 54026 | 13 | begin | 
| 14 | ||
| 15 | ML_file "Tools/coinduction.ML" | |
| 16 | ||
| 17 | end |