changeset 65043 | fd753468786f |
parent 64999 | f8f76a501d25 |
child 66453 | cc19f7ca2ed6 |
--- a/src/HOL/Decision_Procs/Commutative_Ring.thy Wed Feb 22 20:33:53 2017 +0100 +++ b/src/HOL/Decision_Procs/Commutative_Ring.thy Wed Feb 22 20:34:24 2017 +0100 @@ -682,7 +682,7 @@ "0::nat" "1::nat" "2::nat" "3::nat" "0::int" "1::int" "2::int" "3::int" "-1::int" datatypes: polex "(polex * polex) list" int integer num} - (fn p => fn ct => pol_oracle @{context} ct (term_of_pol p)) + (fn ctxt => fn p => fn ct => pol_oracle ctxt ct (term_of_pol p)) end \<close>