src/HOL/PreList.thy
changeset 8756 b03a0b219139
parent 8563 2746bc9a7ef2
child 8840 18b76c137c41
equal deleted inserted replaced
8755:8fdee31b795f 8756:b03a0b219139
     7 basis for theory ToyList in the documentation.
     7 basis for theory ToyList in the documentation.
     8 *)
     8 *)
     9 
     9 
    10 theory PreList =
    10 theory PreList =
    11   Option + WF_Rel + NatBin + Recdef + Record + RelPow + Sexp + Calculation
    11   Option + WF_Rel + NatBin + Recdef + Record + RelPow + Sexp + Calculation
    12   + SVC_Oracle:
    12   + SVC_Oracle
       
    13 files "Integ/NatSimprocs.ML":
    13 
    14 
    14 end
    15 end