src/HOL/Typerep.thy
changeset 38348 cf7b2121ad9d
parent 36176 3fe7e97ccca8
child 38857 97775f3e8722
--- a/src/HOL/Typerep.thy	Wed Aug 11 14:31:40 2010 +0200
+++ b/src/HOL/Typerep.thy	Wed Aug 11 14:31:43 2010 +0200
@@ -56,7 +56,7 @@
     val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, rhs));
   in
     thy
-    |> Theory_Target.instantiation ([tyco], vs, @{sort typerep})
+    |> Class.instantiation ([tyco], vs, @{sort typerep})
     |> `(fn lthy => Syntax.check_term lthy eq)
     |-> (fn eq => Specification.definition (NONE, (Attrib.empty_binding, eq)))
     |> snd