src/HOL/BNF/Coinduction.thy
changeset 54671 d64a4ef26edb
parent 54670 cfb21e03fe2a
parent 54635 30666a281ae3
child 54672 748778ac0ab8
equal deleted inserted replaced
54670:cfb21e03fe2a 54671:d64a4ef26edb
     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