diff -r 2136e4670ad2 -r 5b80eb4fd0f3 src/HOL/Extraction.thy --- a/src/HOL/Extraction.thy Fri Oct 11 21:51:10 2019 +0200 +++ b/src/HOL/Extraction.thy Fri Oct 11 22:01:45 2019 +0200 @@ -17,11 +17,11 @@ [("bool", ([], NONE))] #> Extraction.set_preprocessor (fn thy => Proofterm.rewrite_proof_notypes - ([], RewriteHOLProof.elim_cong :: ProofRewriteRules.rprocs true) o + ([], Rewrite_HOL_Proof.elim_cong :: Proof_Rewrite_Rules.rprocs true) o Proofterm.rewrite_proof thy - (RewriteHOLProof.rews, - ProofRewriteRules.rprocs true @ [ProofRewriteRules.expand_of_class thy]) o - ProofRewriteRules.elim_vars (curry Const \<^const_name>\default\)) + (Rewrite_HOL_Proof.rews, + Proof_Rewrite_Rules.rprocs true @ [Proof_Rewrite_Rules.expand_of_class thy]) o + Proof_Rewrite_Rules.elim_vars (curry Const \<^const_name>\default\)) \ lemmas [extraction_expand] =