src/HOL/Library/comm_ring.ML
changeset 31021 53642251a04f
parent 30510 4120fc59dd85
child 31242 ed40b987a474
equal deleted inserted replaced
31020:9999a77590c3 31021:53642251a04f
    63   | reif_polex T vs (Const (@{const_name Power.power}, _) $ a $ n) =
    63   | reif_polex T vs (Const (@{const_name Power.power}, _) $ a $ n) =
    64       polex_pow T $ reif_polex T vs a $ n
    64       polex_pow T $ reif_polex T vs a $ n
    65   | reif_polex T vs t = polex_pol T $ reif_pol T vs t;
    65   | reif_polex T vs t = polex_pol T $ reif_pol T vs t;
    66 
    66 
    67 (* reification of the equation *)
    67 (* reification of the equation *)
    68 val TFree (_, cr_sort) = @{typ "'a :: {comm_ring, recpower}"};
    68 val cr_sort = @{sort "comm_ring_1"};
    69 
    69 
    70 fun reif_eq thy (eq as Const("op =", Type("fun", [T, _])) $ lhs $ rhs) =
    70 fun reif_eq thy (eq as Const("op =", Type("fun", [T, _])) $ lhs $ rhs) =
    71       if Sign.of_sort thy (T, cr_sort) then
    71       if Sign.of_sort thy (T, cr_sort) then
    72         let
    72         let
    73           val fs = OldTerm.term_frees eq;
    73           val fs = OldTerm.term_frees eq;