src/HOL/Tools/Predicate_Compile/predicate_compile_pred.ML
changeset 59498 50b60f501b05
parent 58963 26bf09b95dda
child 59532 82ab8168d940
equal deleted inserted replaced
59497:0c5cd369a643 59498:50b60f501b05
   133     val ((_, intros), ctxt') = Variable.import true intros ctxt
   133     val ((_, intros), ctxt') = Variable.import true intros ctxt
   134     val (intros', (local_defs, thy')) = (fold_map o fold_map_atoms)
   134     val (intros', (local_defs, thy')) = (fold_map o fold_map_atoms)
   135       (flatten constname) (map prop_of intros) ([], thy)
   135       (flatten constname) (map prop_of intros) ([], thy)
   136     val ctxt'' = Proof_Context.transfer thy' ctxt'
   136     val ctxt'' = Proof_Context.transfer thy' ctxt'
   137     val intros'' =
   137     val intros'' =
   138       map (fn t => Goal.prove ctxt'' [] [] t (fn _ => ALLGOALS Skip_Proof.cheat_tac)) intros'
   138       map (fn t => Goal.prove ctxt'' [] [] t (fn _ => ALLGOALS (Skip_Proof.cheat_tac ctxt''))) intros'
   139       |> Variable.export ctxt'' ctxt
   139       |> Variable.export ctxt'' ctxt
   140   in
   140   in
   141     (intros'', (local_defs, thy'))
   141     (intros'', (local_defs, thy'))
   142   end
   142   end
   143 
   143