author | blanchet |
Wed, 20 Nov 2013 20:45:20 +0100 | |
changeset 54540 | 5d7006e9205e |
parent 54026 | src/HOL/BNF/Coinduction.thy@82d9b2701a03 |
child 54555 | e8c5e95d338b |
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 Inductive begin ML_file "Tools/coinduction.ML" setup Coinduction.setup end