src/HOL/Library/Code_Abstract_Nat.thy
changeset 60801 7664e0916eec
parent 60500 903bb1495239
child 69216 1a52baa70aed
--- a/src/HOL/Library/Code_Abstract_Nat.thy	Mon Jul 27 16:35:12 2015 +0200
+++ b/src/HOL/Library/Code_Abstract_Nat.thy	Mon Jul 27 17:44:55 2015 +0200
@@ -77,7 +77,7 @@
         val thm' =
           Thm.implies_elim
            (Conv.fconv_rule (Thm.beta_conversion true)
-             (Drule.instantiate'
+             (Thm.instantiate'
                [SOME (Thm.ctyp_of_cterm ct)] [SOME (Thm.lambda cv ct),
                  SOME (Thm.lambda cv' (rhs_of thm)), NONE, SOME cv']
                Suc_if_eq)) (Thm.forall_intr cv' thm)