src/HOL/BNF/Coinduction.thy
author traytel
Wed, 02 Oct 2013 11:57:52 +0200
changeset 54026 82d9b2701a03
permissions -rw-r--r--
new coinduction method
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
54026
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     1
(*  Title:      HOL/BNF/Coinduction.thy
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     2
    Author:     Johannes Hölzl, TU Muenchen
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     3
    Author:     Dmitriy Traytel, TU Muenchen
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     4
    Copyright   2013
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     5
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     6
Coinduction method that avoids some boilerplate compared to coinduct.
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     7
*)
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     8
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
     9
header {* Coinduction Method *}
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    10
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    11
theory Coinduction
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    12
imports BNF_Util
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    13
begin
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    14
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    15
ML_file "Tools/coinduction.ML"
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    16
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    17
setup Coinduction.setup
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    18
82d9b2701a03 new coinduction method
traytel
parents:
diff changeset
    19
end