src/HOL/Coinduction.thy
author haftmann
Wed, 08 Jul 2015 14:01:41 +0200
changeset 60688 01488b559910
parent 58889 5b7a9633cfa8
child 60758 d8d85a8172b5
permissions -rw-r--r--
avoid explicit definition of the relation of associated elements in a ring -- prefer explicit normalization instead
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
58889
5b7a9633cfa8 modernized header uniformly as section;
wenzelm
parents: 58814
diff changeset
     9
section {* Coinduction Method *}
54026
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
end