src/HOL/Bali/AxExample.thy
changeset 29258 bce03c644efb
parent 27240 1caa6726168a
child 33965 f57c11db4ad4
--- a/src/HOL/Bali/AxExample.thy	Tue Dec 30 21:46:14 2008 +0100
+++ b/src/HOL/Bali/AxExample.thy	Tue Dec 30 21:46:48 2008 +0100
@@ -41,7 +41,7 @@
 
 ML {*
 fun inst1_tac ctxt s t st =
-  case AList.lookup (op =) (rev (Term.add_varnames (Thm.prop_of st) [])) s of
+  case AList.lookup (op =) (rev (Term.add_var_names (Thm.prop_of st) [])) s of
   SOME i => instantiate_tac ctxt [((s, i), t)] st | NONE => Seq.empty;
 
 val ax_tac =