src/HOL/Coinduction.thy
author wenzelm
Thu, 06 Mar 2014 19:55:08 +0100
changeset 55960 beef468837b1
parent 54555 e8c5e95d338b
child 58814 4c0ad4162cb7
permissions -rw-r--r--
proper position for decode_pos, which is relevant for completion;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
54540
5d7006e9205e moved 'coinduction' proof method to 'HOL'
blanchet
parents: 54026
diff changeset
     1
(*  Title:      HOL/Coinduction.thy
54026
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
54555
e8c5e95d338b rationalize imports
blanchet
parents: 54540
diff changeset
    12
imports Ctr_Sugar
54026
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