| author | blanchet | 
| Wed, 20 Nov 2013 18:58:00 +0100 | |
| changeset 54538 | ba7392b52a7c | 
| parent 54026 | 82d9b2701a03 | 
| permissions | -rw-r--r-- | 
| 54026 | 1 | (* Title: HOL/BNF/Coinduction.thy | 
| 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 | ||
| 9 | header {* Coinduction Method *}
 | |
| 10 | ||
| 11 | theory Coinduction | |
| 12 | imports BNF_Util | |
| 13 | begin | |
| 14 | ||
| 15 | ML_file "Tools/coinduction.ML" | |
| 16 | ||
| 17 | setup Coinduction.setup | |
| 18 | ||
| 19 | end |