NEWS
changeset 44820 7798deb6f8fa
parent 44818 27ba81ad0890
parent 44803 aecfefb05731
child 44826 1120cba9bce4
equal deleted inserted replaced
44819:fe33d6655186 44820:7798deb6f8fa
     1 Isabelle NEWS -- history user-relevant changes
     1 Isabelle NEWS -- history user-relevant changes
     2 ==============================================
     2 ==============================================
     3 
     3 
     4 New in this Isabelle version
     4 New in Isabelle2011-1 (October 2011)
     5 ----------------------------
     5 ------------------------------------
     6 
     6 
     7 *** General ***
     7 *** General ***
     8 
     8 
     9 * Improved Isabelle/jEdit Prover IDE (PIDE), which can be invoked as
     9 * Improved Isabelle/jEdit Prover IDE (PIDE), which can be invoked as
    10 "isabelle jedit" on the command line.
    10 "isabelle jedit" on the command line.
   464 snapshot of the classical context, which can be recovered via
   464 snapshot of the classical context, which can be recovered via
   465 (put_claset HOL_cs) etc.  Type clasimpset has been discontinued.
   465 (put_claset HOL_cs) etc.  Type clasimpset has been discontinued.
   466 INCOMPATIBILITY, classical tactics and derived proof methods require
   466 INCOMPATIBILITY, classical tactics and derived proof methods require
   467 proper Proof.context.
   467 proper Proof.context.
   468 
   468 
       
   469 
       
   470 *** System ***
       
   471 
   469 * Scala layer provides JVM method invocation service for static
   472 * Scala layer provides JVM method invocation service for static
   470 methods of type (String)String, see Invoke_Scala.method in ML.  For
   473 methods of type (String)String, see Invoke_Scala.method in ML.  For
   471 example:
   474 example:
   472 
   475 
   473   Invoke_Scala.method "java.lang.System.getProperty" "java.home"
   476   Invoke_Scala.method "java.lang.System.getProperty" "java.home"
   474 
   477 
   475 Togeter with YXML.string_of_body/parse_body and XML.Encode/Decode this
   478 Togeter with YXML.string_of_body/parse_body and XML.Encode/Decode this
   476 allows to pass structured values between ML and Scala.
   479 allows to pass structured values between ML and Scala.
   477 
   480 
       
   481 * The IsabelleText fonts includes some further glyphs to support the
       
   482 Prover IDE.  Potential INCOMPATIBILITY: users who happen to have
       
   483 installed a local copy (which is normally *not* required) need to
       
   484 delete or update it from ~~/lib/fonts/.
   478 
   485 
   479 
   486 
   480 New in Isabelle2011 (January 2011)
   487 New in Isabelle2011 (January 2011)
   481 ----------------------------------
   488 ----------------------------------
   482 
   489