NEWS
changeset 19211 307dfa3f9e66
parent 19088 7870cf61c4b3
child 19220 05b00acff957
equal deleted inserted replaced
19210:00b01d4445f7 19211:307dfa3f9e66
   326 for example "A -> B" => "Pi A (%_. B)".
   326 for example "A -> B" => "Pi A (%_. B)".
   327 
   327 
   328 
   328 
   329 *** HOL ***
   329 *** HOL ***
   330 
   330 
   331 * Prefer ex1I over ex_ex1I in single-step reasoning, e.g. by the
       
   332 'rule' method.
       
   333 
       
   334 * Alternative iff syntax "A <-> B" for equality on bool (with priority
   331 * Alternative iff syntax "A <-> B" for equality on bool (with priority
   335 25 like -->); output depends on the "iff" print_mode, the default is
   332 25 like -->); output depends on the "iff" print_mode, the default is
   336 "A = B" (with priority 50).
   333 "A = B" (with priority 50).
   337 
   334 
   338 * "LEAST x:A. P" expands to "LEAST x. x:A & P" (input only).
   335 * "LEAST x:A. P" expands to "LEAST x. x:A & P" (input only).
   340 * In the context of the assumption "~(s = t)" the Simplifier rewrites
   337 * In the context of the assumption "~(s = t)" the Simplifier rewrites
   341 "t = s" to False (by simproc "neq_simproc").  For backward
   338 "t = s" to False (by simproc "neq_simproc").  For backward
   342 compatibility this can be disabled by ML "reset use_neq_simproc".
   339 compatibility this can be disabled by ML "reset use_neq_simproc".
   343 
   340 
   344 * "m dvd n" where m and n are numbers is evaluated to True/False by simp.
   341 * "m dvd n" where m and n are numbers is evaluated to True/False by simp.
       
   342 
       
   343 * Theorem Cons_eq_map_conv no longer has attribute `simp'.
       
   344 
       
   345 * Prefer ex1I over ex_ex1I in single-step reasoning, e.g. by the
       
   346 'rule' method.
   345 
   347 
   346 * Tactics 'sat' and 'satx' reimplemented, several improvements: goals
   348 * Tactics 'sat' and 'satx' reimplemented, several improvements: goals
   347 no longer need to be stated as "<prems> ==> False", equivalences (i.e.
   349 no longer need to be stated as "<prems> ==> False", equivalences (i.e.
   348 "=" on type bool) are handled, variable names of the form "lit_<n>"
   350 "=" on type bool) are handled, variable names of the form "lit_<n>"
   349 are no longer reserved, significant speedup.
   351 are no longer reserved, significant speedup.