95 |
95 |
96 * Refined GUI popup for completion: more robust key/mouse event |
96 * Refined GUI popup for completion: more robust key/mouse event |
97 handling and propagation to enclosing text area -- avoid loosing |
97 handling and propagation to enclosing text area -- avoid loosing |
98 keystrokes with slow / remote graphics displays. |
98 keystrokes with slow / remote graphics displays. |
99 |
99 |
|
100 * Completion popup supports both ENTER and TAB (default) to select an |
|
101 item, depending on Isabelle options. |
|
102 |
100 * Refined insertion of completion items wrt. jEdit text: multiple |
103 * Refined insertion of completion items wrt. jEdit text: multiple |
101 selections, rectangular selections, rectangular selection as "tall |
104 selections, rectangular selections, rectangular selection as "tall |
102 caret". |
105 caret". |
103 |
106 |
104 * Integrated spell-checker for document text, comments etc. with |
107 * Integrated spell-checker for document text, comments etc. with |
117 process, without requiring old-fashioned command-line invocation of |
120 process, without requiring old-fashioned command-line invocation of |
118 "isabelle jedit -m MODE". |
121 "isabelle jedit -m MODE". |
119 |
122 |
120 * More support for remote files (e.g. http) using standard Java |
123 * More support for remote files (e.g. http) using standard Java |
121 networking operations instead of jEdit virtual file-systems. |
124 networking operations instead of jEdit virtual file-systems. |
|
125 |
|
126 * Empty editors buffers that are no longer required (e.g.\ via theory |
|
127 imports) are automatically removed from the document model. |
|
128 |
|
129 * Improved monitor panel. |
122 |
130 |
123 * Improved Console/Scala plugin: more uniform scala.Console output, |
131 * Improved Console/Scala plugin: more uniform scala.Console output, |
124 more robust treatment of threads and interrupts. |
132 more robust treatment of threads and interrupts. |
125 |
133 |
126 * Improved management of dockable windows: clarified keyboard focus |
134 * Improved management of dockable windows: clarified keyboard focus |
354 fset_rel ~> rel_fset (in "src/HOL/Library/FSet.thy") |
362 fset_rel ~> rel_fset (in "src/HOL/Library/FSet.thy") |
355 cset_rel ~> rel_cset (in "src/HOL/Library/Countable_Set_Type.thy") |
363 cset_rel ~> rel_cset (in "src/HOL/Library/Countable_Set_Type.thy") |
356 vset ~> rel_vset (in "src/HOL/Library/Quotient_Set.thy") |
364 vset ~> rel_vset (in "src/HOL/Library/Quotient_Set.thy") |
357 |
365 |
358 INCOMPATIBILITY. |
366 INCOMPATIBILITY. |
|
367 |
|
368 * Lifting and Transfer: |
|
369 - a type variable as a raw type is supported |
|
370 - stronger reflexivity prover |
|
371 - rep_eq is always generated by lift_definition |
|
372 - setup for Lifting/Transfer is now automated for BNFs |
|
373 + holds for BNFs that do not contain a dead variable |
|
374 + relator_eq, relator_mono, relator_distr, relator_domain, |
|
375 relator_eq_onp, quot_map, transfer rules for bi_unique, bi_total, |
|
376 right_unique, right_total, left_unique, left_total are proved |
|
377 automatically |
|
378 + definition of a predicator is generated automatically |
|
379 + simplification rules for a predicator definition are proved |
|
380 automatically for datatypes |
|
381 - consolidation of the setup of Lifting/Transfer |
|
382 + property that a relator preservers reflexivity is not needed any |
|
383 more |
|
384 Minor INCOMPATIBILITY. |
|
385 + left_total and left_unique rules are now transfer rules |
|
386 (reflexivity_rule attribute not needed anymore) |
|
387 INCOMPATIBILITY. |
|
388 + Domainp does not have to be a separate assumption in |
|
389 relator_domain theorems (=> more natural statement) |
|
390 INCOMPATIBILITY. |
|
391 - registration of code equations is more robust |
|
392 Potential INCOMPATIBILITY. |
|
393 - respectfulness proof obligation is preprocessed to a more readable |
|
394 form |
|
395 Potential INCOMPATIBILITY. |
|
396 - eq_onp is always unfolded in respectfulness proof obligation |
|
397 Potential INCOMPATIBILITY. |
|
398 - unregister lifting setup for Code_Numeral.integer and |
|
399 Code_Numeral.natural |
|
400 Potential INCOMPATIBILITY. |
|
401 - Lifting.invariant -> eq_onp |
|
402 INCOMPATIBILITY. |
359 |
403 |
360 * New internal SAT solver "cdclite" that produces models and proof |
404 * New internal SAT solver "cdclite" that produces models and proof |
361 traces. This solver replaces the internal SAT solvers "enumerate" and |
405 traces. This solver replaces the internal SAT solvers "enumerate" and |
362 "dpll". Applications that explicitly used one of these two SAT |
406 "dpll". Applications that explicitly used one of these two SAT |
363 solvers should use "cdclite" instead. In addition, "cdclite" is now |
407 solvers should use "cdclite" instead. In addition, "cdclite" is now |
774 * HOL-Library: new theory src/HOL/Library/Tree.thy. |
818 * HOL-Library: new theory src/HOL/Library/Tree.thy. |
775 |
819 |
776 * HOL-Library: removed theory src/HOL/Library/Kleene_Algebra.thy; it |
820 * HOL-Library: removed theory src/HOL/Library/Kleene_Algebra.thy; it |
777 is subsumed by session Kleene_Algebra in AFP. |
821 is subsumed by session Kleene_Algebra in AFP. |
778 |
822 |
|
823 * HOL-Library / theory RBT: various constants and facts are hidden; |
|
824 lifting setup is unregistered. INCOMPATIBILITY. |
|
825 |
779 * HOL-Cardinals: new theory src/HOL/Cardinals/Ordinal_Arithmetic.thy. |
826 * HOL-Cardinals: new theory src/HOL/Cardinals/Ordinal_Arithmetic.thy. |
780 |
827 |
781 * HOL-Word: bit representations prefer type bool over type bit. |
828 * HOL-Word: bit representations prefer type bool over type bit. |
782 INCOMPATIBILITY. |
829 INCOMPATIBILITY. |
783 |
830 |
866 derivative_linear ~> has_derivative_bounded_linear |
913 derivative_linear ~> has_derivative_bounded_linear |
867 derivative_is_linear ~> has_derivative_linear |
914 derivative_is_linear ~> has_derivative_linear |
868 bounded_linear_imp_linear ~> bounded_linear.linear |
915 bounded_linear_imp_linear ~> bounded_linear.linear |
869 |
916 |
870 * HOL-Probability: |
917 * HOL-Probability: |
|
918 - Renamed positive_integral to nn_integral: |
|
919 |
|
920 . Renamed all lemmas "*positive_integral*" to *nn_integral*" |
|
921 positive_integral_positive ~> nn_integral_nonneg |
|
922 |
|
923 . Renamed abbreviation integral\<^sup>P to integral\<^sup>N. |
|
924 |
871 - replaced the Lebesgue integral on real numbers by the more general |
925 - replaced the Lebesgue integral on real numbers by the more general |
872 Bochner integral for functions into a real-normed vector space. |
926 Bochner integral for functions into a real-normed vector space. |
873 |
927 |
874 integral_zero ~> integral_zero / integrable_zero |
928 integral_zero ~> integral_zero / integrable_zero |
875 integral_minus ~> integral_minus / integrable_minus |
929 integral_minus ~> integral_minus / integrable_minus |
880 integral_cmult ~> integral_mult_right / integrable_mult_right |
934 integral_cmult ~> integral_mult_right / integrable_mult_right |
881 integral_triangle_inequality~> integral_norm_bound |
935 integral_triangle_inequality~> integral_norm_bound |
882 integrable_nonneg ~> integrableI_nonneg |
936 integrable_nonneg ~> integrableI_nonneg |
883 integral_positive ~> integral_nonneg_AE |
937 integral_positive ~> integral_nonneg_AE |
884 integrable_abs_iff ~> integrable_abs_cancel |
938 integrable_abs_iff ~> integrable_abs_cancel |
885 positive_integral_lim_INF ~> positive_integral_liminf |
939 positive_integral_lim_INF ~> nn_integral_liminf |
886 lebesgue_real_affine ~> lborel_real_affine |
940 lebesgue_real_affine ~> lborel_real_affine |
887 borel_integral_has_integral ~> has_integral_lebesgue_integral |
941 borel_integral_has_integral ~> has_integral_lebesgue_integral |
888 integral_indicator ~> |
942 integral_indicator ~> |
889 integral_real_indicator / integrable_real_indicator |
943 integral_real_indicator / integrable_real_indicator |
890 positive_integral_fst ~> positive_integral_fst' |
944 positive_integral_fst ~> nn_integral_fst' |
891 positive_integral_fst_measurable ~> positive_integral_fst |
945 positive_integral_fst_measurable ~> nn_integral_fst |
892 positive_integral_snd_measurable ~> positive_integral_snd |
946 positive_integral_snd_measurable ~> nn_integral_snd |
893 |
947 |
894 integrable_fst_measurable ~> |
948 integrable_fst_measurable ~> |
895 integral_fst / integrable_fst / AE_integrable_fst |
949 integral_fst / integrable_fst / AE_integrable_fst |
896 |
950 |
897 integrable_snd_measurable ~> |
951 integrable_snd_measurable ~> |
913 positive_integral_lebesgue_has_integral ~> |
967 positive_integral_lebesgue_has_integral ~> |
914 integral_has_integral_lebesgue_nonneg / |
968 integral_has_integral_lebesgue_nonneg / |
915 integrable_has_integral_lebesgue_nonneg |
969 integrable_has_integral_lebesgue_nonneg |
916 |
970 |
917 lebesgue_integral_real_affine ~> |
971 lebesgue_integral_real_affine ~> |
918 positive_integral_real_affine |
972 nn_integral_real_affine |
919 |
973 |
920 has_integral_iff_positive_integral_lborel ~> |
974 has_integral_iff_positive_integral_lborel ~> |
921 integral_has_integral_nonneg / integrable_has_integral_nonneg |
975 integral_has_integral_nonneg / integrable_has_integral_nonneg |
922 |
976 |
923 The following theorems where removed: |
977 The following theorems where removed: |
927 lebesgue_integral_cmult |
981 lebesgue_integral_cmult |
928 lebesgue_integral_multc |
982 lebesgue_integral_multc |
929 lebesgue_integral_cmult_nonneg |
983 lebesgue_integral_cmult_nonneg |
930 integral_cmul_indicator |
984 integral_cmul_indicator |
931 integral_real |
985 integral_real |
932 |
|
933 - Renamed positive_integral to nn_integral: |
|
934 |
|
935 . Renamed all lemmas "*positive_integral*" to *nn_integral*" |
|
936 positive_integral_positive ~> nn_integral_nonneg |
|
937 |
|
938 . Renamed abbreviation integral\<^sup>P to integral\<^sup>N. |
|
939 |
986 |
940 - Formalized properties about exponentially, Erlang, and normal |
987 - Formalized properties about exponentially, Erlang, and normal |
941 distributed random variables. |
988 distributed random variables. |
942 |
989 |
943 * HOL-Decision_Procs: Separate command 'approximate' for approximative |
990 * HOL-Decision_Procs: Separate command 'approximate' for approximative |