src/Tools/isac/ProgLang/ProgLang.thy
changeset 59423 e1b34eb27309
parent 59412 3bd4be5666de
child 59424 406681ebe781
equal deleted inserted replaced
59422:e1c3d997d665 59423:e1b34eb27309
     6 theory ProgLang imports Script
     6 theory ProgLang imports Script
     7 begin
     7 begin
     8 
     8 
     9 ML_file "~~/src/Tools/isac/ProgLang/scrtools.sml"
     9 ML_file "~~/src/Tools/isac/ProgLang/scrtools.sml"
    10 
    10 
       
    11 partial_function (tailrec)
       
    12   solve_equation :: "bool \<Rightarrow> real \<Rightarrow> bool list "
       
    13 where
       
    14   "solve_equation eq bdv = [eq, eq, eq]"
       
    15 ML {*
       
    16 @{term solve_equation}
       
    17 *}
       
    18 
       
    19 thm "solve_equation.simps"
       
    20 ML {*
       
    21 val thm = @{thm solve_equation.simps}
       
    22 *} ML {*
       
    23 Thm.prop_of thm
       
    24 *} ML {*
       
    25 *}
       
    26 
    11 ML {*
    27 ML {*
    12 *} ML {*
    28 *} ML {*
    13 *}
    29 *}
    14 end
    30 end