src/Tools/isac/IsacKnowledge/LogExp.thy
branchisac-update-Isa09-2
changeset 37947 22235e4dbe5f
parent 37906 e2b23ba9df13
equal deleted inserted replaced
37946:a28b5fc129b7 37947:22235e4dbe5f
     1 (* all outcommented in order to demonstrate authoring:
       
     2    WN071203
       
     3 remove_thy"LogExp";
       
     4 use_thy_only"IsacKnowledge/LogExp";
       
     5 use_thy_only"IsacKnowledge/Isac";
       
     6 *)
       
     7 LogExp = PolyEq + 
       
     8 
       
     9 consts
       
    10 
       
    11   ln     :: "real => real"
       
    12   exp    :: "real => real"         ("E'_ ^^^ _" 80)
       
    13 
       
    14 (*--------------------------------------------------*) 
       
    15   alog   :: "[real, real] => real" ("_ log _" 90)
       
    16 
       
    17   (*Script-names*)
       
    18   Solve'_log    :: "[bool,real,        bool list] \
       
    19 				   \=> bool list"
       
    20                   ("((Script Solve'_log (_ _=))//(_))" 9)
       
    21 
       
    22 rules
       
    23 
       
    24   equality_pow    "0 < a ==> (l = r) = (a^^^l = a^^^r)"
       
    25   (* this is what students   ^^^^^^^... are told to do *)
       
    26   equality_power  "((a log b) = c) = (a^^^(a log b) = a^^^c)"
       
    27   exp_invers_log  "a^^^(a log b) = b"
       
    28 (*---------------------------------------------------*)
       
    29 
       
    30 end