src/HOL/Bali/Basis.thy
changeset 59755 f8d164ab0dc1
parent 59498 50b60f501b05
child 61424 c3658c18b7bc
--- a/src/HOL/Bali/Basis.thy	Thu Mar 19 17:25:57 2015 +0100
+++ b/src/HOL/Bali/Basis.thy	Thu Mar 19 22:30:57 2015 +0100
@@ -180,7 +180,7 @@
 fun sum3_instantiate ctxt thm =
   map (fn s =>
     simplify (ctxt delsimps @{thms not_None_eq})
-      (Rule_Insts.read_instantiate ctxt [(("t", 0), "In" ^ s ^ " x")] ["x"] thm))
+      (Rule_Insts.read_instantiate ctxt [((("t", 0), Position.none), "In" ^ s ^ " x")] ["x"] thm))
     ["1l","2","3","1r"]
 *}
 (* e.g. lemmas is_stmt_rews = is_stmt_def [of "In1l x", simplified] *)