src/HOL/PreList.thy
changeset 14430 5cb24165a2e1
parent 14125 bf8edef6c1f1
child 14577 dbb95b825244
equal deleted inserted replaced
14429:0fce2d8bce0f 14430:5cb24165a2e1
     7 header{*A Basis for Building the Theory of Lists*}
     7 header{*A Basis for Building the Theory of Lists*}
     8 
     8 
     9 (*Is defined separately to serve as a basis for theory ToyList in the
     9 (*Is defined separately to serve as a basis for theory ToyList in the
    10 documentation.*)
    10 documentation.*)
    11 
    11 
    12 theory PreList = Wellfounded_Relations + Presburger + Recdef + Relation_Power:
    12 theory PreList =
       
    13     Wellfounded_Relations + Presburger + Recdef + Relation_Power + Parity:
    13 
    14 
    14 (*belongs to theory Wellfounded_Recursion*)
    15 (*belongs to theory Wellfounded_Recursion*)
    15 lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf]
    16 lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf]
    16 
    17 
    17 end
    18 end