src/HOL/ex/SVC_Oracle.thy
changeset 48891 c0eafbd55de3
parent 46218 ecf6375e2abb
child 52131 366fa32ee2a3
equal deleted inserted replaced
48890:d72ca5742f80 48891:c0eafbd55de3
     7 
     7 
     8 header {* Installing an oracle for SVC (Stanford Validity Checker) *}
     8 header {* Installing an oracle for SVC (Stanford Validity Checker) *}
     9 
     9 
    10 theory SVC_Oracle
    10 theory SVC_Oracle
    11 imports Main
    11 imports Main
    12 uses "svc_funcs.ML"
       
    13 begin
    12 begin
       
    13 
       
    14 ML_file "svc_funcs.ML"
    14 
    15 
    15 consts
    16 consts
    16   iff_keep :: "[bool, bool] => bool"
    17   iff_keep :: "[bool, bool] => bool"
    17   iff_unfold :: "[bool, bool] => bool"
    18   iff_unfold :: "[bool, bool] => bool"
    18 
    19