adapted ProofContext.infer_type;
authorwenzelm
Thu, 29 Apr 2010 17:15:23 +0200
changeset 36506 6b56e679d9ff
parent 36505 79c1d2bbe5a9
child 36507 c966a1aab860
adapted ProofContext.infer_type;
src/HOL/Statespace/state_space.ML
--- a/src/HOL/Statespace/state_space.ML	Thu Apr 29 16:55:22 2010 +0200
+++ b/src/HOL/Statespace/state_space.ML	Thu Apr 29 17:15:23 2010 +0200
@@ -198,7 +198,7 @@
   if Variable.is_fixed ctxt name orelse Variable.is_declared ctxt name
   then
     let val n' = lookupI (op =) (Variable.fixes_of ctxt) name
-    in SOME (Free (n',ProofContext.infer_type ctxt n')) end
+    in SOME (Free (n',ProofContext.infer_type ctxt (n', dummyT))) end
   else NONE
 
 
@@ -430,7 +430,7 @@
           let
             fun upd (n,v) =
               let
-                val nT = ProofContext.infer_type (Local_Theory.target_of lthy) n
+                val nT = ProofContext.infer_type (Local_Theory.target_of lthy) (n, dummyT)
               in Context.proof_map
                   (update_declinfo (Morphism.term phi (Free (n,nT)),v))
               end;