src/ZF/Induct/Acc.thy
changeset 58871 c399ae4b836f
parent 58623 2db1df2c8467
child 60770 240563fbf41d
equal deleted inserted replaced
58870:e2c0d8ef29cb 58871:c399ae4b836f
     1 (*  Title:      ZF/Induct/Acc.thy
     1 (*  Title:      ZF/Induct/Acc.thy
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Copyright   1994  University of Cambridge
     3     Copyright   1994  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header {* The accessible part of a relation *}
     6 section {* The accessible part of a relation *}
     7 
     7 
     8 theory Acc imports Main begin
     8 theory Acc imports Main begin
     9 
     9 
    10 text {*
    10 text {*
    11   Inductive definition of @{text "acc(r)"}; see @{cite "paulin-tlca"}.
    11   Inductive definition of @{text "acc(r)"}; see @{cite "paulin-tlca"}.