1 Isabelle NEWS -- history of user-relevant changes
2 =================================================
4 (Note: Isabelle/jEdit shows a tree-view of this file in Sidekick.)
7 New in this Isabelle version
8 ----------------------------
12 * Toplevel theorem statements have been simplified as follows:
15 schematic_lemma ~> schematic_goal
16 schematic_theorem ~> schematic_goal
17 schematic_corollary ~> schematic_goal
19 Command-line tool "isabelle update_theorems" updates theory sources
22 * Toplevel theorem statement 'proposition' is another alias for
25 * HTML presentation uses the standard IsabelleText font and Unicode
26 rendering of Isabelle symbols like Isabelle/Scala/jEdit. The former
27 print mode "HTML" looses its special meaning.
30 *** Prover IDE -- Isabelle/Scala/jEdit ***
32 * Improved scheduling for urgent print tasks (e.g. command state output,
33 interactive queries) wrt. long-running background tasks.
35 * IDE support for the source-level debugger of Poly/ML, to work with
36 Isabelle/ML and official Standard ML. Configuration option "ML_debugger"
37 and commands 'ML_file_debug', 'ML_file_no_debug', 'SML_file_debug',
38 'SML_file_no_debug' control compilation of sources with debugging
39 information. The Debugger panel allows to set breakpoints (via context
40 menu), step through stopped threads, evaluate local ML expressions etc.
41 At least one Debugger view needs to be active to have any effect on the
44 * The main Isabelle executable is managed as single-instance Desktop
45 application uniformly on all platforms: Linux, Windows, Mac OS X.
47 * The text overview column (status of errors, warnings etc.) is updated
48 asynchronously, leading to much better editor reactivity. Moreover, the
49 full document node content is taken into account.
51 * The State panel manages explicit proof state output, with jEdit action
52 "isabelle.update-state" (shortcut S+ENTER) to trigger update according
53 to cursor position. Option "editor_output_state" controls implicit proof
54 state output in the Output panel: suppressing this reduces resource
55 requirements of prover time and GUI space.
58 *** Document preparation ***
60 * Isabelle control symbols for markup and formatting:
62 \<^smallskip> \smallskip
66 \<^item> \item (itemize)
67 \<^enum> \item (enumeration)
72 * Command 'obtain' binds term abbreviations (via 'is' patterns) in the
73 proof body as well, abstracted over relevant parameters.
75 * Improved type-inference for theorem statement 'obtains': separate
76 parameter scope for of each clause.
78 * Term abbreviations via 'is' patterns also work for schematic
79 statements: result is abstracted over unknowns.
81 * Local goals ('have', 'show', 'hence', 'thus') allow structured
82 statements like fixes/assumes/shows in theorem specifications, but the
83 notation is postfix with keywords 'if' (or 'when') and 'for'. For
88 for x :: 'a and y :: 'a
91 The local assumptions are bound to the name "that". The result is
92 exported from context of the statement as usual. The above roughly
93 corresponds to a raw proof block like this:
96 fix x :: 'a and y :: 'a
97 assume that: "A x" "B y"
102 The keyword 'when' may be used instead of 'if', to indicate 'presume'
103 instead of 'assume' above.
105 * The meaning of 'show' with Pure rule statements has changed: premises
106 are treated in the sense of 'assume', instead of 'presume'. This means,
107 a goal like "\<And>x. A x \<Longrightarrow> B x \<Longrightarrow> C x" can be solved completely as follows:
109 show "\<And>x. A x \<Longrightarrow> B x \<Longrightarrow> C x"
113 show "C x" if "A x" "B x" for x
115 Rare INCOMPATIBILITY, the old behaviour may be recovered as follows:
117 show "C x" when "A x" "B x" for x
119 * New command 'supply' supports fact definitions during goal refinement
122 * New command 'consider' states rules for generalized elimination and
123 case splitting. This is like a toplevel statement "theorem obtains" used
124 within a proof body; or like a multi-branch 'obtain' without activation
125 of the local context elements yet.
127 * Proof method "cases" allows to specify the rule as first entry of
128 chained facts. This is particularly useful with 'consider':
130 consider (a) A | (b) B | (c) C <proof>
134 then show ?thesis <proof>
137 then show ?thesis <proof>
140 then show ?thesis <proof>
143 * Command 'case' allows fact name and attribute specification like this:
146 case a [attributes]: (c xs)
148 Facts that are introduced by invoking the case context are uniformly
149 qualified by "a"; the same name is used for the cumulative fact. The old
150 form "case (c xs) [attributes]" is no longer supported. Rare
151 INCOMPATIBILITY, need to adapt uses of case facts in exotic situations,
152 and always put attributes in front.
154 * The standard proof method of commands 'proof' and '..' is now called
155 "standard" to make semantically clear what it is; the old name "default"
156 is still available as legacy for some time. Documentation now explains
157 '..' more accurately as "by standard" instead of "by rule".
159 * Command 'subgoal' allows to impose some structure on backward
160 refinements, to avoid proof scripts degenerating into long of 'apply'
161 sequences. Further explanations and examples are given in the isar-ref
164 * Proof method "goal_cases" turns the current subgoals into cases within
165 the context; the conclusion is bound to variable ?case in each case. For
168 lemma "\<And>x. A x \<Longrightarrow> B x \<Longrightarrow> C x"
169 and "\<And>y z. U y \<Longrightarrow> V z \<Longrightarrow> W y z"
172 then show ?case using \<open>A x\<close> \<open>B x\<close> sorry
175 then show ?case using \<open>U y\<close> \<open>V z\<close> sorry
178 lemma "\<And>x. A x \<Longrightarrow> B x \<Longrightarrow> C x"
179 and "\<And>y z. U y \<Longrightarrow> V z \<Longrightarrow> W y z"
182 then show ?case using prems sorry
185 then show ?case using prems sorry
188 * The undocumented feature of implicit cases goal1, goal2, goal3, etc.
189 is marked as legacy, and will be removed eventually. The proof method
190 "goals" achieves a similar effect within regular Isar; often it can be
191 done more adequately by other means (e.g. 'consider').
193 * Nesting of Isar goal structure has been clarified: the context after
194 the initial backwards refinement is retained for the whole proof, within
195 all its context sections (as indicated via 'next'). This is e.g.
196 relevant for 'using', 'including', 'supply':
198 have "A \<and> A" if a: A for A
206 * Method "sleep" succeeds after a real-time delay (in seconds). This is
207 occasionally useful for demonstration and testing purposes.
212 * Command 'print_definitions' prints dependencies of definitional
213 specifications. This functionality used to be part of 'print_theory'.
215 * The vacuous fact "TERM x" may be established "by fact" or as `TERM x`
216 as well, not just "by this" or "." as before.
218 * Configuration option rule_insts_schematic has been discontinued
219 (intermediate legacy feature in Isabelle2015). INCOMPATIBILITY.
221 * Abbreviations in type classes now carry proper sort constraint.
222 Rare INCOMPATIBILITY in situations where the previous misbehaviour
225 * Refinement of user-space type system in type classes: pseudo-local
226 operations behave more similar to abbreviations. Potential
227 INCOMPATIBILITY in exotic situations.
232 * Combinator to represent case distinction on products is named "case_prod",
233 uniformly, discontinuing any input aliasses. Very popular theorem aliasses
236 PairE ~> prod.exhaust
237 Pair_eq ~> prod.inject
238 pair_collapse ~> prod.collapse
239 Pair_fst_snd_eq ~> prod_eq_iff
240 split_twice ~> prod.case_distrib
241 split_weak_cong ~> prod.case_cong_weak
242 split_split ~> prod.split
243 split_split_asm ~> prod.split_asm
246 splitI2 ~> case_prodI2
247 splitI2' ~> case_prodI2'
249 splitE' ~> case_prodE'
250 split_pair ~> case_prod_Pair
251 split_eta ~> case_prod_eta
252 split_comp ~> case_prod_comp
253 mem_splitI ~> mem_case_prodI
254 mem_splitI2 ~> mem_case_prodI2
255 mem_splitE ~> mem_case_prodE
256 The_split ~> The_case_prod
257 cond_split_eta ~> cond_case_prod_eta
258 Collect_split_in_rel_leE ~> Collect_case_prod_in_rel_leE
259 Collect_split_in_rel_leI ~> Collect_case_prod_in_rel_leI
260 in_rel_Collect_split_eq ~> in_rel_Collect_case_prod_eq
261 Collect_split_Grp_eqD ~> Collect_case_prod_Grp_eqD
262 Collect_split_Grp_inD ~> Collect_case_prod_Grp_in
263 Domain_Collect_split ~> Domain_Collect_case_prod
264 Image_Collect_split ~> Image_Collect_case_prod
265 Range_Collect_split ~> Range_Collect_case_prod
266 Eps_split ~> Eps_case_prod
267 Eps_split_eq ~> Eps_case_prod_eq
268 split_rsp ~> case_prod_rsp
269 curry_split ~> curry_case_prod
270 split_curry ~> case_prod_curry
271 Changes in structure HOLogic:
272 split_const ~> case_prod_const
273 mk_split ~> mk_case_prod
274 mk_psplits ~> mk_ptupleabs
275 strip_psplits ~> strip_ptupleabs
278 * Commands 'inductive' and 'inductive_set' work better when names for
279 intro rules are omitted: the "cases" and "induct" rules no longer
280 declare empty case_names, but no case_names at all. This allows to use
281 numbered cases in proofs, without requiring method "goal_cases".
283 * The 'typedef' command has been upgraded from a partially checked
284 "axiomatization", to a full definitional specification that takes the
285 global collection of overloaded constant / type definitions into
286 account. Type definitions with open dependencies on overloaded
287 definitions need to be specified as "typedef (overloaded)". This
288 provides extra robustness in theory construction. Rare INCOMPATIBILITY.
290 * Qualification of various formal entities in the libraries is done more
291 uniformly via "context begin qualified definition ... end" instead of
292 old-style "hide_const (open) ...". Consequently, both the defined
293 constant and its defining fact become qualified, e.g. Option.is_none and
294 Option.is_none_def. Occasional INCOMPATIBILITY in applications.
296 * Some old and rarely used ASCII replacement syntax has been removed.
297 INCOMPATIBILITY, standard syntax with symbols should be used instead.
298 The subsequent commands help to reproduce the old forms, e.g. to
299 simplify porting old theories:
301 type_notation Map.map (infixr "~=>" 0)
302 notation Map.map_comp (infixl "o'_m" 55)
304 type_notation FinFun.finfun ("(_ =>f /_)" [22, 21] 21)
306 notation FuncSet.funcset (infixr "->" 60)
307 notation FuncSet.extensional_funcset (infixr "->\<^sub>E" 60)
309 notation Omega_Words_Fun.conc (infixr "conc" 65)
311 notation Preorder.equiv ("op ~~")
312 and Preorder.equiv ("(_/ ~~ _)" [51, 51] 50)
314 * The alternative notation "\<Colon>" for type and sort constraints has been
315 removed: in LaTeX document output it looks the same as "::".
316 INCOMPATIBILITY, use plain "::" instead.
318 * Theory Map: lemma map_of_is_SomeD was a clone of map_of_SomeD and has
319 been removed. INCOMPATIBILITY.
321 * Quickcheck setup for finite sets.
323 * Discontinued simp_legacy_precond. Potential INCOMPATIBILITY.
326 - The MaSh relevance filter has been sped up.
327 - Proof reconstruction has been improved, to minimize the incidence of
328 cases where Sledgehammer gives a proof that does not work.
329 - Auto Sledgehammer now minimizes and preplays the results.
330 - Handle Vampire 4.0 proof output without raising exception.
331 - Eliminated "MASH" environment variable. Use the "MaSh" option in
332 Isabelle/jEdit instead. INCOMPATIBILITY.
333 - Eliminated obsolete "blocking" option and related subcommands.
336 - Fixed soundness bug in translation of "finite" predicate.
337 - Fixed soundness bug in "destroy_constrs" optimization.
338 - Removed "check_potential" and "check_genuine" options.
339 - Eliminated obsolete "blocking" option.
341 * New (co)datatype package:
342 - New commands "lift_bnf" and "copy_bnf" for lifting (copying) a BNF
343 structure on the raw type to an abstract type defined using typedef.
344 - Always generate "case_transfer" theorem.
347 - new methods for interactive debugging of 'transfer' and
348 'transfer_prover': 'transfer_start', 'transfer_step', 'transfer_end',
349 'transfer_prover_start' and 'transfer_prover_end'.
351 * Division on integers is bootstrapped directly from division on
352 naturals and uses generic numeral algorithm for computations.
353 Slight INCOMPATIBILITY, simproc numeral_divmod replaces and generalizes
354 former simprocs binary_int_div and binary_int_mod
356 * Tightened specification of class semiring_no_zero_divisors. Slight
359 * Class algebraic_semidom introduces common algebraic notions of
360 integral (semi)domains, particularly units. Although
361 logically subsumed by fields, is is not a super class of these
362 in order not to burden fields with notions that are trivial there.
364 * Class normalization_semidom specifies canonical representants
365 for equivalence classes of associated elements in an integral
366 (semi)domain. This formalizes associated elements as well.
368 * Abstract specification of gcd/lcm operations in classes semiring_gcd,
369 semiring_Gcd, semiring_Lcd. Minor INCOMPATIBILITY: facts gcd_nat.commute
370 and gcd_int.commute are subsumed by gcd.commute, as well as gcd_nat.assoc
371 and gcd_int.assoc by gcd.assoc.
373 * Former constants Fields.divide (_ / _) and Divides.div (_ div _)
374 are logically unified to Rings.divide in syntactic type class
375 Rings.divide, with infix syntax (_ div _). Infix syntax (_ / _)
376 for field division is added later as abbreviation in class Fields.inverse.
377 INCOMPATIBILITY, instantiations must refer to Rings.divide rather
378 than the former separate constants, hence infix syntax (_ / _) is usually
379 not available during instantiation.
382 - Renamed multiset inclusion operators:
384 \<subset> ~> \<subset>#
387 \<subseteq> ~> \<subseteq>#
389 - "'a multiset" is no longer an instance of the "order",
390 "ordered_ab_semigroup_add_imp_le", "ordered_cancel_comm_monoid_diff",
391 "semilattice_inf", and "semilattice_sup" type classes. The theorems
392 previously provided by these type classes (directly or indirectly)
393 are now available through the "subset_mset" interpretation
394 (e.g. add_mono ~> subset_mset.add_mono).
396 - Renamed conversions:
398 multiset_of_set ~> mset_set
402 mset_le_def ~> subseteq_mset_def
403 mset_less_def ~> subset_mset_def
404 less_eq_multiset.rep_eq ~> subseteq_mset_def
406 - Removed lemmas generated by lift_definition:
407 less_eq_multiset.abs_eq, less_eq_multiset.rsp less_eq_multiset.transfer
411 * Multivariate_Analysis/Cauchy_Integral_Thm: Complex path integrals and Cauchy's integral theorem,
412 ported from HOL Light
414 * Theory Library/Old_Recdef: discontinued obsolete 'defer_recdef'
415 command. Minor INCOMPATIBILITY, use 'function' instead.
417 * Recursive function definitions ('fun', 'function', 'partial_function')
418 no longer expose the low-level "_def" facts of the internal
419 construction. INCOMPATIBILITY, enable option "function_defs" in the
420 context for rare situations where these facts are really needed.
422 * Imperative_HOL: obsolete theory Legacy_Mrec has been removed.
424 * Library/Omega_Words_Fun: Infinite words modeled as functions nat => 'a.
429 * The auxiliary module Pure/display.ML has been eliminated. Its
430 elementary thm print operations are now in Pure/more_thm.ML and thus
431 called Thm.pretty_thm, Thm.string_of_thm etc. INCOMPATIBILITY.
433 * Simproc programming interfaces have been simplified:
434 Simplifier.make_simproc and Simplifier.define_simproc supersede various
435 forms of Simplifier.mk_simproc, Simplifier.simproc_global etc. Note that
436 term patterns for the left-hand sides are specified with implicitly
437 fixed variables, like top-level theorem statements. INCOMPATIBILITY.
439 * Instantiation rules have been re-organized as follows:
441 Thm.instantiate (*low-level instantiation with named arguments*)
442 Thm.instantiate' (*version with positional arguments*)
444 Drule.infer_instantiate (*instantiation with type inference*)
445 Drule.infer_instantiate' (*version with positional arguments*)
447 The LHS only requires variable specifications, instead of full terms.
448 Old cterm_instantiate is superseded by infer_instantiate.
449 INCOMPATIBILITY, need to re-adjust some ML names and types accordingly.
451 * Old tactic shorthands atac, rtac, etac, dtac, ftac have been
452 discontinued. INCOMPATIBILITY, use regular assume_tac, resolve_tac etc.
453 instead (with proper context).
455 * Thm.instantiate (and derivatives) no longer require the LHS of the
456 instantiation to be certified: plain variables are given directly.
458 * Subgoal.SUBPROOF and Subgoal.FOCUS combinators use anonymous
459 quasi-bound variables (like the Simplifier), instead of accidentally
460 named local fixes. This has the potential to improve stability of proof
461 tools, but can also cause INCOMPATIBILITY for tools that don't observe
462 the proof context discipline.
467 * Property values in etc/symbols may contain spaces, if written with the
468 replacement character "␣" (Unicode point 0x2324). For example:
470 \<star> code: 0x0022c6 group: operator font: Deja␣Vu␣Sans␣Mono
472 * Command-line tool "isabelle jedit_client" allows to connect to already
473 running Isabelle/jEdit process. This achieves the effect of
474 single-instance applications seen on common GUI desktops.
476 * Command-line tool "isabelle update_then" expands old Isar command
482 This syntax is more orthogonal and improves readability and
483 maintainability of proofs.
485 * Poly/ML default platform architecture may be changed from 32bit to
486 64bit via system option ML_system_64. A system restart (and rebuild)
487 is required after change.
489 * Poly/ML 5.5.3 runs natively on x86-windows and x86_64-windows,
490 which both allow larger heap space than former x86-cygwin.
492 * Java runtime environment for x86_64-windows allows to use larger heap
495 * Java runtime options are determined separately for 32bit vs. 64bit
496 platforms as follows.
498 - Isabelle desktop application: platform-specific files that are
499 associated with the main app bundle
501 - isabelle jedit: settings
502 JEDIT_JAVA_SYSTEM_OPTIONS
503 JEDIT_JAVA_OPTIONS32 vs. JEDIT_JAVA_OPTIONS64
505 - isabelle build: settings
506 ISABELLE_BUILD_JAVA_OPTIONS32 vs. ISABELLE_BUILD_JAVA_OPTIONS64
508 * Bash shell function "jvmpath" has been renamed to "platform_path": it
509 is relevant both for Poly/ML and JVM processes.
513 New in Isabelle2015 (May 2015)
514 ------------------------------
518 * Local theory specification commands may have a 'private' or
519 'qualified' modifier to restrict name space accesses to the local scope,
520 as provided by some "context begin ... end" block. For example:
525 private definition ...
528 qualified definition ...
536 * Command 'experiment' opens an anonymous locale context with private
539 * Command 'notepad' requires proper nesting of begin/end and its proof
540 structure in the body: 'oops' is no longer supported here. Minor
541 INCOMPATIBILITY, use 'sorry' instead.
543 * Command 'named_theorems' declares a dynamic fact within the context,
544 together with an attribute to maintain the content incrementally. This
545 supersedes functor Named_Thms in Isabelle/ML, but with a subtle change
546 of semantics due to external visual order vs. internal reverse order.
548 * 'find_theorems': search patterns which are abstractions are
549 schematically expanded before search. Search results match the naive
550 expectation more closely, particularly wrt. abbreviations.
553 * Commands 'method_setup' and 'attribute_setup' now work within a local
556 * Outer syntax commands are managed authentically within the theory
557 context, without implicit global state. Potential for accidental
558 INCOMPATIBILITY, make sure that required theories are really imported.
560 * Historical command-line terminator ";" is no longer accepted (and
561 already used differently in Isar). Minor INCOMPATIBILITY, use "isabelle
562 update_semicolons" to remove obsolete semicolons from old theory
565 * Structural composition of proof methods (meth1; meth2) in Isar
566 corresponds to (tac1 THEN_ALL_NEW tac2) in ML.
568 * The Eisbach proof method language allows to define new proof methods
569 by combining existing ones with their usual syntax. The "match" proof
570 method provides basic fact/term matching in addition to
571 premise/conclusion matching through Subgoal.focus, and binds fact names
572 from matches as well as term patterns within matches. The Isabelle
573 documentation provides an entry "eisbach" for the Eisbach User Manual.
574 Sources and various examples are in ~~/src/HOL/Eisbach/.
577 *** Prover IDE -- Isabelle/Scala/jEdit ***
579 * Improved folding mode "isabelle" based on Isar syntax. Alternatively,
580 the "sidekick" mode may be used for document structure.
582 * Extended bracket matching based on Isar language structure. System
583 option jedit_structure_limit determines maximum number of lines to scan
586 * Support for BibTeX files: context menu, context-sensitive token
587 marker, SideKick parser.
589 * Document antiquotation @{cite} provides formal markup, which is
590 interpreted semi-formally based on .bib files that happen to be open in
591 the editor (hyperlinks, completion etc.).
593 * Less waste of vertical space via negative line spacing (see Global
594 Options / Text Area).
596 * Improved graphview panel with optional output of PNG or PDF, for
597 display of 'thy_deps', 'class_deps' etc.
599 * The commands 'thy_deps' and 'class_deps' allow optional bounds to
600 restrict the visualized hierarchy.
602 * Improved scheduling for asynchronous print commands (e.g. provers
603 managed by the Sledgehammer panel) wrt. ongoing document processing.
606 *** Document preparation ***
608 * Document markup commands 'chapter', 'section', 'subsection',
609 'subsubsection', 'text', 'txt', 'text_raw' work uniformly in any
610 context, even before the initial 'theory' command. Obsolete proof
611 commands 'sect', 'subsect', 'subsubsect', 'txt_raw' have been
612 discontinued, use 'section', 'subsection', 'subsubsection', 'text_raw'
613 instead. The old 'header' command is still retained for some time, but
614 should be replaced by 'chapter', 'section' etc. (using "isabelle
615 update_header"). Minor INCOMPATIBILITY.
617 * Official support for "tt" style variants, via \isatt{...} or
618 \begin{isabellett}...\end{isabellett}. The somewhat fragile \verb or
619 verbatim environment of LaTeX is no longer used. This allows @{ML} etc.
620 as argument to other macros (such as footnotes).
622 * Document antiquotation @{verbatim} prints ASCII text literally in "tt"
625 * Discontinued obsolete option "document_graph": session_graph.pdf is
626 produced unconditionally for HTML browser_info and PDF-LaTeX document.
628 * Diagnostic commands and document markup commands within a proof do not
629 affect the command tag for output. Thus commands like 'thm' are subject
630 to proof document structure, and no longer "stick out" accidentally.
631 Commands 'text' and 'txt' merely differ in the LaTeX style, not their
632 tags. Potential INCOMPATIBILITY in exotic situations.
634 * System option "pretty_margin" is superseded by "thy_output_margin",
635 which is also accessible via document antiquotation option "margin".
636 Only the margin for document output may be changed, but not the global
637 pretty printing: that is 76 for plain console output, and adapted
638 dynamically in GUI front-ends. Implementations of document
639 antiquotations need to observe the margin explicitly according to
640 Thy_Output.string_of_margin. Minor INCOMPATIBILITY.
642 * Specification of 'document_files' in the session ROOT file is
643 mandatory for document preparation. The legacy mode with implicit
644 copying of the document/ directory is no longer supported. Minor
650 * Proof methods with explicit instantiation ("rule_tac", "subgoal_tac"
651 etc.) allow an optional context of local variables ('for' declaration):
652 these variables become schematic in the instantiated theorem; this
653 behaviour is analogous to 'for' in attributes "where" and "of".
654 Configuration option rule_insts_schematic (default false) controls use
655 of schematic variables outside the context. Minor INCOMPATIBILITY,
656 declare rule_insts_schematic = true temporarily and update to use local
657 variable declarations or dummy patterns instead.
659 * Explicit instantiation via attributes "where", "of", and proof methods
660 "rule_tac" with derivatives like "subgoal_tac" etc. admit dummy patterns
661 ("_") that stand for anonymous local variables.
663 * Generated schematic variables in standard format of exported facts are
664 incremented to avoid material in the proof context. Rare
665 INCOMPATIBILITY, explicit instantiation sometimes needs to refer to
668 * Lexical separation of signed and unsigned numerals: categories "num"
669 and "float" are unsigned. INCOMPATIBILITY: subtle change in precedence
670 of numeral signs, particularly in expressions involving infix syntax
673 * Old inner token category "xnum" has been discontinued. Potential
674 INCOMPATIBILITY for exotic syntax: may use mixfix grammar with "num"
675 token category instead.
680 * New (co)datatype package:
681 - The 'datatype_new' command has been renamed 'datatype'. The old
682 command of that name is now called 'old_datatype' and is provided
683 by "~~/src/HOL/Library/Old_Datatype.thy". See
684 'isabelle doc datatypes' for information on porting.
687 disc_corec ~> corec_disc
688 disc_corec_iff ~> corec_disc_iff
689 disc_exclude ~> distinct_disc
690 disc_exhaust ~> exhaust_disc
691 disc_map_iff ~> map_disc_iff
692 sel_corec ~> corec_sel
693 sel_exhaust ~> exhaust_sel
696 sel_split ~> split_sel
697 sel_split_asm ~> split_sel_asm
698 strong_coinduct ~> coinduct_strong
699 weak_case_cong ~> case_cong_weak
701 - The "no_code" option to "free_constructors", "datatype_new", and
702 "codatatype" has been renamed "plugins del: code".
704 - The rules "set_empty" have been removed. They are easy
705 consequences of other set rules "by auto".
707 - The rule "set_cases" is now registered with the "[cases set]"
708 attribute. This can influence the behavior of the "cases" proof
709 method when more than one case rule is applicable (e.g., an
710 assumption is of the form "w : set ws" and the method "cases w"
711 is invoked). The solution is to specify the case rule explicitly
712 (e.g. "cases w rule: widget.exhaust").
715 BNF_Comp ~> BNF_Composition
716 BNF_FP_Base ~> BNF_Fixpoint_Base
717 BNF_GFP ~> BNF_Greatest_Fixpoint
718 BNF_LFP ~> BNF_Least_Fixpoint
719 BNF_Constructions_on_Wellorders ~> BNF_Wellorder_Constructions
720 Cardinals/Constructions_on_Wellorders ~> Cardinals/Wellorder_Constructions
722 - Lifting and Transfer setup for basic HOL types sum and prod (also
723 option) is now performed by the BNF package. Theories Lifting_Sum,
724 Lifting_Product and Lifting_Option from Main became obsolete and
725 were removed. Changed definitions of the relators rel_prod and
726 rel_sum (using inductive).
727 INCOMPATIBILITY: use rel_prod.simps and rel_sum.simps instead
728 of rel_prod_def and rel_sum_def.
729 Minor INCOMPATIBILITY: (rarely used by name) transfer theorem names
730 changed (e.g. map_prod_transfer ~> prod.map_transfer).
731 - Parametricity theorems for map functions, relators, set functions,
732 constructors, case combinators, discriminators, selectors and
733 (co)recursors are automatically proved and registered as transfer
736 * Old datatype package:
737 - The old 'datatype' command has been renamed 'old_datatype', and
738 'rep_datatype' has been renamed 'old_rep_datatype'. They are
739 provided by "~~/src/HOL/Library/Old_Datatype.thy". See
740 'isabelle doc datatypes' for information on porting.
743 weak_case_cong ~> case_cong_weak
746 ~~/src/HOL/Datatype.thy ~> ~~/src/HOL/Library/Old_Datatype.thy
750 - Fixed soundness bug related to the strict and non-strict subset
754 - CVC4 is now included with Isabelle instead of CVC3 and run by
756 - Z3 is now always enabled by default, now that it is fully open
757 source. The "z3_non_commercial" option is discontinued.
758 - Minimization is now always enabled by default.
761 - Proof reconstruction, both one-liners and Isar, has been
762 dramatically improved.
763 - Improved support for CVC4 and veriT.
765 * Old and new SMT modules:
766 - The old 'smt' method has been renamed 'old_smt' and moved to
767 'src/HOL/Library/Old_SMT.thy'. It is provided for compatibility,
768 until applications have been ported to use the new 'smt' method. For
769 the method to work, an older version of Z3 (e.g. Z3 3.2 or 4.0) must
770 be installed, and the environment variable "OLD_Z3_SOLVER" must
773 - The 'smt2' method has been renamed 'smt'.
775 - New option 'smt_reconstruction_step_timeout' to limit the
776 reconstruction time of Z3 proof steps in the new 'smt' method.
777 - New option 'smt_statistics' to display statistics of the new 'smt'
778 method, especially runtime statistics of Z3 proof reconstruction.
780 * Lifting: command 'lift_definition' allows to execute lifted constants
781 that have as a return type a datatype containing a subtype. This
782 overcomes long-time limitations in the area of code generation and
783 lifting, and avoids tedious workarounds.
785 * Command and antiquotation "value" provide different evaluation slots
786 (again), where the previous strategy (NBE after ML) serves as default.
787 Minor INCOMPATIBILITY.
789 * Add NO_MATCH-simproc, allows to check for syntactic non-equality.
791 * field_simps: Use NO_MATCH-simproc for distribution rules, to avoid
792 non-termination in case of distributing a division. With this change
793 field_simps is in some cases slightly less powerful, if it fails try to
794 add algebra_simps, or use divide_simps. Minor INCOMPATIBILITY.
796 * Separate class no_zero_divisors has been given up in favour of fully
797 algebraic semiring_no_zero_divisors. INCOMPATIBILITY.
799 * Class linordered_semidom really requires no zero divisors.
802 * Classes division_ring, field and linordered_field always demand
803 "inverse 0 = 0". Given up separate classes division_ring_inverse_zero,
804 field_inverse_zero and linordered_field_inverse_zero. INCOMPATIBILITY.
806 * Classes cancel_ab_semigroup_add / cancel_monoid_add specify explicit
807 additive inverse operation. INCOMPATIBILITY.
809 * Complex powers and square roots. The functions "ln" and "powr" are now
810 overloaded for types real and complex, and 0 powr y = 0 by definition.
811 INCOMPATIBILITY: type constraints may be necessary.
813 * The functions "sin" and "cos" are now defined for any type of sort
814 "{real_normed_algebra_1,banach}" type, so in particular on "real" and
815 "complex" uniformly. Minor INCOMPATIBILITY: type constraints may be
818 * New library of properties of the complex transcendental functions sin,
819 cos, tan, exp, Ln, Arctan, Arcsin, Arccos. Ported from HOL Light.
821 * The factorial function, "fact", now has type "nat => 'a" (of a sort
822 that admits numeric types including nat, int, real and complex.
823 INCOMPATIBILITY: an expression such as "fact 3 = 6" may require a type
824 constraint, and the combination "real (fact k)" is likely to be
825 unsatisfactory. If a type conversion is still necessary, then use
826 "of_nat (fact k)" or "real_of_nat (fact k)".
828 * Removed functions "natfloor" and "natceiling", use "nat o floor" and
829 "nat o ceiling" instead. A few of the lemmas have been retained and
830 adapted: in their names "natfloor"/"natceiling" has been replaced by
831 "nat_floor"/"nat_ceiling".
833 * Qualified some duplicated fact names required for boostrapping the
834 type class hierarchy:
835 ab_add_uminus_conv_diff ~> diff_conv_add_uminus
836 field_inverse_zero ~> inverse_zero
837 field_divide_inverse ~> divide_inverse
838 field_inverse ~> left_inverse
839 Minor INCOMPATIBILITY.
841 * Eliminated fact duplicates:
842 mult_less_imp_less_right ~> mult_right_less_imp_less
843 mult_less_imp_less_left ~> mult_left_less_imp_less
844 Minor INCOMPATIBILITY.
846 * Fact consolidation: even_less_0_iff is subsumed by
847 double_add_less_zero_iff_single_add_less_zero (simp by default anyway).
849 * Generalized and consolidated some theorems concerning divsibility:
850 dvd_reduce ~> dvd_add_triv_right_iff
851 dvd_plus_eq_right ~> dvd_add_right_iff
852 dvd_plus_eq_left ~> dvd_add_left_iff
853 Minor INCOMPATIBILITY.
855 * "even" and "odd" are mere abbreviations for "2 dvd _" and "~ 2 dvd _"
856 and part of theory Main.
857 even_def ~> even_iff_mod_2_eq_zero
860 * Lemma name consolidation: divide_Numeral1 ~> divide_numeral_1. Minor
863 * Bootstrap of listsum as special case of abstract product over lists.
865 listsum_def ~> listsum.eq_foldr
868 * Product over lists via constant "listprod".
870 * Theory List: renamed drop_Suc_conv_tl and nth_drop' to
873 * New infrastructure for compiling, running, evaluating and testing
874 generated code in target languages in HOL/Library/Code_Test. See
875 HOL/Codegenerator_Test/Code_Test* for examples.
878 - Introduced "replicate_mset" operation.
879 - Introduced alternative characterizations of the multiset ordering in
880 "Library/Multiset_Order".
881 - Renamed multiset ordering:
884 \<subset># ~> #\<subset>#
885 \<subseteq># ~> #\<subseteq>#
887 - Introduced abbreviations for ill-named multiset operations:
888 <#, \<subset># abbreviate < (strict subset)
889 <=#, \<le>#, \<subseteq># abbreviate <= (subset or equal)
892 in_multiset_of ~> in_multiset_in_set
893 Multiset.fold ~> fold_mset
894 Multiset.filter ~> filter_mset
896 - Removed mcard, is equal to size.
900 elem_multiset_of_set [simp, intro]
901 comp_fun_commute_plus_mset [simp]
902 comp_fun_commute.fold_mset_insert [OF comp_fun_commute_plus_mset, simp]
903 in_mset_fold_plus_iff [iff]
904 set_of_Union_mset [simp]
905 in_Union_mset_iff [iff]
908 * Library/Sum_of_Squares: simplified and improved "sos" method. Always
909 use local CSDP executable, which is much faster than the NEOS server.
910 The "sos_cert" functionality is invoked as "sos" with additional
911 argument. Minor INCOMPATIBILITY.
913 * HOL-Decision_Procs: New counterexample generator quickcheck
914 [approximation] for inequalities of transcendental functions. Uses
915 hardware floating point arithmetic to randomly discover potential
916 counterexamples. Counterexamples are certified with the "approximation"
917 method. See HOL/Decision_Procs/ex/Approximation_Quickcheck_Ex.thy for
920 * HOL-Probability: Reworked measurability prover
921 - applies destructor rules repeatedly
922 - removed application splitting (replaced by destructor rule)
923 - added congruence rules to rewrite measure spaces under the sets
926 * New proof method "rewrite" (in theory ~~/src/HOL/Library/Rewrite) for
927 single-step rewriting with subterm selection based on patterns.
932 * Subtle change of name space policy: undeclared entries are now
933 considered inaccessible, instead of accessible via the fully-qualified
934 internal name. This mainly affects Name_Space.intern (and derivatives),
935 which may produce an unexpected Long_Name.hidden prefix. Note that
936 contemporary applications use the strict Name_Space.check (and
937 derivatives) instead, which is not affected by the change. Potential
938 INCOMPATIBILITY in rare applications of Name_Space.intern.
940 * Subtle change of error semantics of Toplevel.proof_of: regular user
941 ERROR instead of internal Toplevel.UNDEF.
943 * Basic combinators map, fold, fold_map, split_list, apply are available
944 as parameterized antiquotations, e.g. @{map 4} for lists of quadruples.
946 * Renamed "pairself" to "apply2", in accordance to @{apply 2}.
949 * Former combinators NAMED_CRITICAL and CRITICAL for central critical
950 sections have been discontinued, in favour of the more elementary
951 Multithreading.synchronized and its high-level derivative
952 Synchronized.var (which is usually sufficient in applications). Subtle
953 INCOMPATIBILITY: synchronized access needs to be atomic and cannot be
956 * Synchronized.value (ML) is actually synchronized (as in Scala): subtle
957 change of semantics with minimal potential for INCOMPATIBILITY.
959 * The main operations to certify logical entities are Thm.ctyp_of and
960 Thm.cterm_of with a local context; old-style global theory variants are
961 available as Thm.global_ctyp_of and Thm.global_cterm_of.
964 * Elementary operations in module Thm are no longer pervasive.
965 INCOMPATIBILITY, need to use qualified Thm.prop_of, Thm.cterm_of,
968 * Proper context for various elementary tactics: assume_tac,
969 resolve_tac, eresolve_tac, dresolve_tac, forward_tac, match_tac,
970 compose_tac, Splitter.split_tac etc. INCOMPATIBILITY.
972 * Tactical PARALLEL_ALLGOALS is the most common way to refer to
975 * Goal.prove_multi is superseded by the fully general Goal.prove_common,
976 which also allows to specify a fork priority.
978 * Antiquotation @{command_spec "COMMAND"} is superseded by
979 @{command_keyword COMMAND} (usually without quotes and with PIDE
980 markup). Minor INCOMPATIBILITY.
982 * Cartouches within ML sources are turned into values of type
983 Input.source (with formal position information).
988 * The Isabelle tool "update_cartouches" changes theory files to use
989 cartouches instead of old-style {* verbatim *} or `alt_string` tokens.
991 * The Isabelle tool "build" provides new options -X, -k, -x.
993 * Discontinued old-fashioned "codegen" tool. Code generation can always
994 be externally triggered using an appropriate ROOT file plus a
995 corresponding theory. Parametrization is possible using environment
996 variables, or ML snippets in the most extreme cases. Minor
999 * JVM system property "isabelle.threads" determines size of Scala thread
1000 pool, like Isabelle system option "threads" for ML.
1002 * JVM system property "isabelle.laf" determines the default Swing
1003 look-and-feel, via internal class name or symbolic name as in the jEdit
1004 menu Global Options / Appearance.
1006 * Support for Proof General and Isar TTY loop has been discontinued.
1007 Minor INCOMPATIBILITY, use standard PIDE infrastructure instead.
1011 New in Isabelle2014 (August 2014)
1012 ---------------------------------
1016 * Support for official Standard ML within the Isabelle context.
1017 Command 'SML_file' reads and evaluates the given Standard ML file.
1018 Toplevel bindings are stored within the theory context; the initial
1019 environment is restricted to the Standard ML implementation of
1020 Poly/ML, without the add-ons of Isabelle/ML. Commands 'SML_import'
1021 and 'SML_export' allow to exchange toplevel bindings between the two
1022 separate environments. See also ~~/src/Tools/SML/Examples.thy for
1025 * Standard tactics and proof methods such as "clarsimp", "auto" and
1026 "safe" now preserve equality hypotheses "x = expr" where x is a free
1027 variable. Locale assumptions and chained facts containing "x"
1028 continue to be useful. The new method "hypsubst_thin" and the
1029 configuration option "hypsubst_thin" (within the attribute name space)
1030 restore the previous behavior. INCOMPATIBILITY, especially where
1031 induction is done after these methods or when the names of free and
1032 bound variables clash. As first approximation, old proofs may be
1033 repaired by "using [[hypsubst_thin = true]]" in the critical spot.
1035 * More static checking of proof methods, which allows the system to
1036 form a closure over the concrete syntax. Method arguments should be
1037 processed in the original proof context as far as possible, before
1038 operating on the goal state. In any case, the standard discipline for
1039 subgoal-addressing needs to be observed: no subgoals or a subgoal
1040 number that is out of range produces an empty result sequence, not an
1041 exception. Potential INCOMPATIBILITY for non-conformant tactical
1044 * Lexical syntax (inner and outer) supports text cartouches with
1045 arbitrary nesting, and without escapes of quotes etc. The Prover IDE
1046 supports input via ` (backquote).
1048 * The outer syntax categories "text" (for formal comments and document
1049 markup commands) and "altstring" (for literal fact references) allow
1050 cartouches as well, in addition to the traditional mix of quotations.
1052 * Syntax of document antiquotation @{rail} now uses \<newline> instead
1053 of "\\", to avoid the optical illusion of escaped backslash within
1054 string token. General renovation of its syntax using text cartouches.
1055 Minor INCOMPATIBILITY.
1057 * Discontinued legacy_isub_isup, which was a temporary workaround for
1058 Isabelle/ML in Isabelle2013-1. The prover process no longer accepts
1059 old identifier syntax with \<^isub> or \<^isup>. Potential
1062 * Document antiquotation @{url} produces markup for the given URL,
1063 which results in an active hyperlink within the text.
1065 * Document antiquotation @{file_unchecked} is like @{file}, but does
1066 not check existence within the file-system.
1068 * Updated and extended manuals: codegen, datatypes, implementation,
1069 isar-ref, jedit, system.
1072 *** Prover IDE -- Isabelle/Scala/jEdit ***
1074 * Improved Document panel: simplified interaction where every single
1075 mouse click (re)opens document via desktop environment or as jEdit
1078 * Support for Navigator plugin (with toolbar buttons), with connection
1081 * Auxiliary files ('ML_file' etc.) are managed by the Prover IDE.
1082 Open text buffers take precedence over copies within the file-system.
1084 * Improved support for Isabelle/ML, with jEdit mode "isabelle-ml" for
1087 * Improved syntactic and semantic completion mechanism, with simple
1088 templates, completion language context, name-space completion,
1089 file-name completion, spell-checker completion.
1091 * Refined GUI popup for completion: more robust key/mouse event
1092 handling and propagation to enclosing text area -- avoid loosing
1093 keystrokes with slow / remote graphics displays.
1095 * Completion popup supports both ENTER and TAB (default) to select an
1096 item, depending on Isabelle options.
1098 * Refined insertion of completion items wrt. jEdit text: multiple
1099 selections, rectangular selections, rectangular selection as "tall
1102 * Integrated spell-checker for document text, comments etc. with
1103 completion popup and context-menu.
1105 * More general "Query" panel supersedes "Find" panel, with GUI access
1106 to commands 'find_theorems' and 'find_consts', as well as print
1107 operations for the context. Minor incompatibility in keyboard
1108 shortcuts etc.: replace action isabelle-find by isabelle-query.
1110 * Search field for all output panels ("Output", "Query", "Info" etc.)
1111 to highlight text via regular expression.
1113 * Option "jedit_print_mode" (see also "Plugin Options / Isabelle /
1114 General") allows to specify additional print modes for the prover
1115 process, without requiring old-fashioned command-line invocation of
1116 "isabelle jedit -m MODE".
1118 * More support for remote files (e.g. http) using standard Java
1119 networking operations instead of jEdit virtual file-systems.
1121 * Empty editors buffers that are no longer required (e.g.\ via theory
1122 imports) are automatically removed from the document model.
1124 * Improved monitor panel.
1126 * Improved Console/Scala plugin: more uniform scala.Console output,
1127 more robust treatment of threads and interrupts.
1129 * Improved management of dockable windows: clarified keyboard focus
1130 and window placement wrt. main editor view; optional menu item to
1131 "Detach" a copy where this makes sense.
1133 * New Simplifier Trace panel provides an interactive view of the
1134 simplification process, enabled by the "simp_trace_new" attribute
1140 * Low-level type-class commands 'classes', 'classrel', 'arities' have
1141 been discontinued to avoid the danger of non-trivial axiomatization
1142 that is not immediately visible. INCOMPATIBILITY, use regular
1143 'instance' command with proof. The required OFCLASS(...) theorem
1144 might be postulated via 'axiomatization' beforehand, or the proof
1145 finished trivially if the underlying class definition is made vacuous
1146 (without any assumptions). See also Isabelle/ML operations
1147 Axclass.class_axiomatization, Axclass.classrel_axiomatization,
1148 Axclass.arity_axiomatization.
1150 * Basic constants of Pure use more conventional names and are always
1151 qualified. Rare INCOMPATIBILITY, but with potentially serious
1152 consequences, notably for tools in Isabelle/ML. The following
1153 renaming needs to be applied:
1159 dummy_pattern ~> Pure.dummy_pattern
1161 Systematic porting works by using the following theory setup on a
1162 *previous* Isabelle version to introduce the new name accesses for the
1168 |> Sign.const_alias (Binding.qualify true "Pure" @{binding eq}) "=="
1169 |> Sign.const_alias (Binding.qualify true "Pure" @{binding imp}) "==>"
1170 |> Sign.const_alias (Binding.qualify true "Pure" @{binding all}) "all"
1171 |> Sign.restore_naming thy
1174 Thus ML antiquotations like @{const_name Pure.eq} may be used already.
1175 Later the application is moved to the current Isabelle version, and
1176 the auxiliary aliases are deleted.
1178 * Attributes "where" and "of" allow an optional context of local
1179 variables ('for' declaration): these variables become schematic in the
1180 instantiated theorem.
1182 * Obsolete attribute "standard" has been discontinued (legacy since
1183 Isabelle2012). Potential INCOMPATIBILITY, use explicit 'for' context
1184 where instantiations with schematic variables are intended (for
1185 declaration commands like 'lemmas' or attributes like "of"). The
1186 following temporary definition may help to port old applications:
1188 attribute_setup standard =
1189 "Scan.succeed (Thm.rule_attribute (K Drule.export_without_context))"
1191 * More thorough check of proof context for goal statements and
1192 attributed fact expressions (concerning background theory, declared
1193 hyps). Potential INCOMPATIBILITY, tools need to observe standard
1194 context discipline. See also Assumption.add_assumes and the more
1195 primitive Thm.assume_hyps.
1197 * Inner syntax token language allows regular quoted strings "..."
1198 (only makes sense in practice, if outer syntax is delimited
1199 differently, e.g. via cartouches).
1201 * Command 'print_term_bindings' supersedes 'print_binds' for clarity,
1202 but the latter is retained some time as Proof General legacy.
1204 * Code generator preprocessor: explicit control of simp tracing on a
1205 per-constant basis. See attribute "code_preproc".
1210 * Code generator: enforce case of identifiers only for strict target
1211 language requirements. INCOMPATIBILITY.
1213 * Code generator: explicit proof contexts in many ML interfaces.
1216 * Code generator: minimize exported identifiers by default. Minor
1219 * Code generation for SML and OCaml: dropped arcane "no_signatures"
1220 option. Minor INCOMPATIBILITY.
1222 * "declare [[code abort: ...]]" replaces "code_abort ...".
1225 * "declare [[code drop: ...]]" drops all code equations associated
1226 with the given constants.
1228 * Code generations are provided for make, fields, extend and truncate
1229 operations on records.
1231 * Command and antiquotation "value" are now hardcoded against nbe and
1232 ML. Minor INCOMPATIBILITY.
1234 * Renamed command 'enriched_type' to 'functor'. INCOMPATIBILITY.
1236 * The symbol "\<newline>" may be used within char or string literals
1237 to represent (Char Nibble0 NibbleA), i.e. ASCII newline.
1239 * Qualified String.implode and String.explode. INCOMPATIBILITY.
1241 * Simplifier: Enhanced solver of preconditions of rewrite rules can
1242 now deal with conjunctions. For help with converting proofs, the old
1243 behaviour of the simplifier can be restored like this: declare/using
1244 [[simp_legacy_precond]]. This configuration option will disappear
1245 again in the future. INCOMPATIBILITY.
1247 * Simproc "finite_Collect" is no longer enabled by default, due to
1248 spurious crashes and other surprises. Potential INCOMPATIBILITY.
1250 * Moved new (co)datatype package and its dependencies from session
1251 "HOL-BNF" to "HOL". The commands 'bnf', 'wrap_free_constructors',
1252 'datatype_new', 'codatatype', 'primcorec', 'primcorecursive' are now
1253 part of theory "Main".
1256 FunDef.thy ~> Fun_Def.thy (and Fun_Def_Base.thy)
1257 Library/Wfrec.thy ~> Wfrec.thy
1258 Library/Zorn.thy ~> Zorn.thy
1259 Cardinals/Order_Relation.thy ~> Order_Relation.thy
1260 Library/Order_Union.thy ~> Cardinals/Order_Union.thy
1261 Cardinals/Cardinal_Arithmetic_Base.thy ~> BNF_Cardinal_Arithmetic.thy
1262 Cardinals/Cardinal_Order_Relation_Base.thy ~> BNF_Cardinal_Order_Relation.thy
1263 Cardinals/Constructions_on_Wellorders_Base.thy ~> BNF_Constructions_on_Wellorders.thy
1264 Cardinals/Wellorder_Embedding_Base.thy ~> BNF_Wellorder_Embedding.thy
1265 Cardinals/Wellorder_Relation_Base.thy ~> BNF_Wellorder_Relation.thy
1266 BNF/Ctr_Sugar.thy ~> Ctr_Sugar.thy
1267 BNF/Basic_BNFs.thy ~> Basic_BNFs.thy
1268 BNF/BNF_Comp.thy ~> BNF_Comp.thy
1269 BNF/BNF_Def.thy ~> BNF_Def.thy
1270 BNF/BNF_FP_Base.thy ~> BNF_FP_Base.thy
1271 BNF/BNF_GFP.thy ~> BNF_GFP.thy
1272 BNF/BNF_LFP.thy ~> BNF_LFP.thy
1273 BNF/BNF_Util.thy ~> BNF_Util.thy
1274 BNF/Coinduction.thy ~> Coinduction.thy
1275 BNF/More_BNFs.thy ~> Library/More_BNFs.thy
1276 BNF/Countable_Type.thy ~> Library/Countable_Set_Type.thy
1277 BNF/Examples/* ~> BNF_Examples/*
1280 Wellorder_Extension.thy (split from Zorn.thy)
1281 Library/Cardinal_Notations.thy
1282 Library/BNF_Axomatization.thy
1283 BNF_Examples/Misc_Primcorec.thy
1284 BNF_Examples/Stream_Processor.thy
1286 Discontinued theories:
1288 BNF/Equiv_Relations_More.thy
1292 * New (co)datatype package:
1293 - Command 'primcorec' is fully implemented.
1294 - Command 'datatype_new' generates size functions ("size_xxx" and
1295 "size") as required by 'fun'.
1296 - BNFs are integrated with the Lifting tool and new-style
1297 (co)datatypes with Transfer.
1299 datatype_new_compat ~> datatype_compat
1300 primrec_new ~> primrec
1301 wrap_free_constructors ~> free_constructors
1303 - The generated constants "xxx_case" and "xxx_rec" have been renamed
1304 "case_xxx" and "rec_xxx" (e.g., "prod_case" ~> "case_prod").
1306 - The constant "xxx_(un)fold" and related theorems are no longer
1307 generated. Use "xxx_(co)rec" or define "xxx_(un)fold" manually
1308 using "prim(co)rec".
1310 - No discriminators are generated for nullary constructors by
1311 default, eliminating the need for the odd "=:" syntax.
1313 - No discriminators or selectors are generated by default by
1314 "datatype_new", unless custom names are specified or the new
1315 "discs_sels" option is passed.
1318 * Old datatype package:
1319 - The generated theorems "xxx.cases" and "xxx.recs" have been
1320 renamed "xxx.case" and "xxx.rec" (e.g., "sum.cases" ->
1321 "sum.case"). INCOMPATIBILITY.
1322 - The generated constants "xxx_case", "xxx_rec", and "xxx_size" have
1323 been renamed "case_xxx", "rec_xxx", and "size_xxx" (e.g.,
1324 "prod_case" ~> "case_prod"). INCOMPATIBILITY.
1326 * The types "'a list" and "'a option", their set and map functions,
1327 their relators, and their selectors are now produced using the new
1328 BNF-based datatype package.
1331 Option.set ~> set_option
1332 Option.map ~> map_option
1333 option_rel ~> rel_option
1336 set_def ~> set_rec[abs_def]
1337 map_def ~> map_rec[abs_def]
1338 Option.map_def ~> map_option_case[abs_def] (with "case_option" instead of "rec_option")
1339 option.recs ~> option.rec
1340 list_all2_def ~> list_all2_iff
1341 set.simps ~> set_simps (or the slightly different "list.set")
1342 map.simps ~> list.map
1343 hd.simps ~> list.sel(1)
1344 tl.simps ~> list.sel(2-3)
1345 the.simps ~> option.sel
1349 * The following map functions and relators have been renamed:
1351 map_pair ~> map_prod
1352 prod_rel ~> rel_prod
1356 filter_rel ~> rel_filter
1357 fset_rel ~> rel_fset (in "src/HOL/Library/FSet.thy")
1358 cset_rel ~> rel_cset (in "src/HOL/Library/Countable_Set_Type.thy")
1359 vset ~> rel_vset (in "src/HOL/Library/Quotient_Set.thy")
1363 * Lifting and Transfer:
1364 - a type variable as a raw type is supported
1365 - stronger reflexivity prover
1366 - rep_eq is always generated by lift_definition
1367 - setup for Lifting/Transfer is now automated for BNFs
1368 + holds for BNFs that do not contain a dead variable
1369 + relator_eq, relator_mono, relator_distr, relator_domain,
1370 relator_eq_onp, quot_map, transfer rules for bi_unique, bi_total,
1371 right_unique, right_total, left_unique, left_total are proved
1373 + definition of a predicator is generated automatically
1374 + simplification rules for a predicator definition are proved
1375 automatically for datatypes
1376 - consolidation of the setup of Lifting/Transfer
1377 + property that a relator preservers reflexivity is not needed any
1379 Minor INCOMPATIBILITY.
1380 + left_total and left_unique rules are now transfer rules
1381 (reflexivity_rule attribute not needed anymore)
1383 + Domainp does not have to be a separate assumption in
1384 relator_domain theorems (=> more natural statement)
1386 - registration of code equations is more robust
1387 Potential INCOMPATIBILITY.
1388 - respectfulness proof obligation is preprocessed to a more readable
1390 Potential INCOMPATIBILITY.
1391 - eq_onp is always unfolded in respectfulness proof obligation
1392 Potential INCOMPATIBILITY.
1393 - unregister lifting setup for Code_Numeral.integer and
1394 Code_Numeral.natural
1395 Potential INCOMPATIBILITY.
1396 - Lifting.invariant -> eq_onp
1399 * New internal SAT solver "cdclite" that produces models and proof
1400 traces. This solver replaces the internal SAT solvers "enumerate" and
1401 "dpll". Applications that explicitly used one of these two SAT
1402 solvers should use "cdclite" instead. In addition, "cdclite" is now
1403 the default SAT solver for the "sat" and "satx" proof methods and
1404 corresponding tactics; the old default can be restored using "declare
1405 [[sat_solver = zchaff_with_proofs]]". Minor INCOMPATIBILITY.
1407 * SMT module: A new version of the SMT module, temporarily called
1408 "SMT2", uses SMT-LIB 2 and supports recent versions of Z3 (e.g.,
1409 4.3). The new proof method is called "smt2". CVC3 and CVC4 are also
1410 supported as oracles. Yices is no longer supported, because no version
1411 of the solver can handle both SMT-LIB 2 and quantifiers.
1413 * Activation of Z3 now works via "z3_non_commercial" system option
1414 (without requiring restart), instead of former settings variable
1415 "Z3_NON_COMMERCIAL". The option can be edited in Isabelle/jEdit menu
1416 Plugin Options / Isabelle / General.
1419 - Z3 can now produce Isar proofs.
1421 . New SML-based learning algorithms eliminate the dependency on
1422 Python and increase performance and reliability.
1423 . MaSh and MeSh are now used by default together with the
1424 traditional MePo (Meng-Paulson) relevance filter. To disable
1425 MaSh, set the "MaSh" system option in Isabelle/jEdit Plugin
1426 Options / Isabelle / General to "none".
1430 isar_compress ~> compress
1435 * Removed solvers remote_cvc3 and remote_z3. Use cvc3 and z3 instead.
1438 - Fixed soundness bug whereby mutually recursive datatypes could
1439 take infinite values.
1440 - Fixed soundness bug with low-level number functions such as
1441 "Abs_Integ" and "Rep_Integ".
1442 - Removed "std" option.
1443 - Renamed "show_datatypes" to "show_types" and "hide_datatypes" to
1446 * Metis: Removed legacy proof method 'metisFT'. Use 'metis
1447 (full_types)' instead. INCOMPATIBILITY.
1449 * Try0: Added 'algebra' and 'meson' to the set of proof methods.
1451 * Adjustion of INF and SUP operations:
1452 - Elongated constants INFI and SUPR to INFIMUM and SUPREMUM.
1453 - Consolidated theorem names containing INFI and SUPR: have INF and
1454 SUP instead uniformly.
1455 - More aggressive normalization of expressions involving INF and Inf
1457 - INF_image and SUP_image do not unfold composition.
1458 - Dropped facts INF_comp, SUP_comp.
1459 - Default congruence rules strong_INF_cong and strong_SUP_cong, with
1460 simplifier implication in premises. Generalize and replace former
1465 * SUP and INF generalized to conditionally_complete_lattice.
1467 * Swapped orientation of facts image_comp and vimage_comp:
1469 image_compose ~> image_comp [symmetric]
1470 image_comp ~> image_comp [symmetric]
1471 vimage_compose ~> vimage_comp [symmetric]
1472 vimage_comp ~> vimage_comp [symmetric]
1476 * Theory reorganization: split of Big_Operators.thy into
1477 Groups_Big.thy and Lattices_Big.thy.
1479 * Consolidated some facts about big group operators:
1481 setsum_0' ~> setsum.neutral
1482 setsum_0 ~> setsum.neutral_const
1483 setsum_addf ~> setsum.distrib
1484 setsum_cartesian_product ~> setsum.cartesian_product
1485 setsum_cases ~> setsum.If_cases
1486 setsum_commute ~> setsum.commute
1487 setsum_cong ~> setsum.cong
1488 setsum_delta ~> setsum.delta
1489 setsum_delta' ~> setsum.delta'
1490 setsum_diff1' ~> setsum.remove
1491 setsum_empty ~> setsum.empty
1492 setsum_infinite ~> setsum.infinite
1493 setsum_insert ~> setsum.insert
1494 setsum_inter_restrict'' ~> setsum.inter_filter
1495 setsum_mono_zero_cong_left ~> setsum.mono_neutral_cong_left
1496 setsum_mono_zero_cong_right ~> setsum.mono_neutral_cong_right
1497 setsum_mono_zero_left ~> setsum.mono_neutral_left
1498 setsum_mono_zero_right ~> setsum.mono_neutral_right
1499 setsum_reindex ~> setsum.reindex
1500 setsum_reindex_cong ~> setsum.reindex_cong
1501 setsum_reindex_nonzero ~> setsum.reindex_nontrivial
1502 setsum_restrict_set ~> setsum.inter_restrict
1503 setsum_Plus ~> setsum.Plus
1504 setsum_setsum_restrict ~> setsum.commute_restrict
1505 setsum_Sigma ~> setsum.Sigma
1506 setsum_subset_diff ~> setsum.subset_diff
1507 setsum_Un_disjoint ~> setsum.union_disjoint
1508 setsum_UN_disjoint ~> setsum.UNION_disjoint
1509 setsum_Un_Int ~> setsum.union_inter
1510 setsum_Union_disjoint ~> setsum.Union_disjoint
1511 setsum_UNION_zero ~> setsum.Union_comp
1512 setsum_Un_zero ~> setsum.union_inter_neutral
1513 strong_setprod_cong ~> setprod.strong_cong
1514 strong_setsum_cong ~> setsum.strong_cong
1515 setprod_1' ~> setprod.neutral
1516 setprod_1 ~> setprod.neutral_const
1517 setprod_cartesian_product ~> setprod.cartesian_product
1518 setprod_cong ~> setprod.cong
1519 setprod_delta ~> setprod.delta
1520 setprod_delta' ~> setprod.delta'
1521 setprod_empty ~> setprod.empty
1522 setprod_infinite ~> setprod.infinite
1523 setprod_insert ~> setprod.insert
1524 setprod_mono_one_cong_left ~> setprod.mono_neutral_cong_left
1525 setprod_mono_one_cong_right ~> setprod.mono_neutral_cong_right
1526 setprod_mono_one_left ~> setprod.mono_neutral_left
1527 setprod_mono_one_right ~> setprod.mono_neutral_right
1528 setprod_reindex ~> setprod.reindex
1529 setprod_reindex_cong ~> setprod.reindex_cong
1530 setprod_reindex_nonzero ~> setprod.reindex_nontrivial
1531 setprod_Sigma ~> setprod.Sigma
1532 setprod_subset_diff ~> setprod.subset_diff
1533 setprod_timesf ~> setprod.distrib
1534 setprod_Un2 ~> setprod.union_diff2
1535 setprod_Un_disjoint ~> setprod.union_disjoint
1536 setprod_UN_disjoint ~> setprod.UNION_disjoint
1537 setprod_Un_Int ~> setprod.union_inter
1538 setprod_Union_disjoint ~> setprod.Union_disjoint
1539 setprod_Un_one ~> setprod.union_inter_neutral
1541 Dropped setsum_cong2 (simple variant of setsum.cong).
1542 Dropped setsum_inter_restrict' (simple variant of setsum.inter_restrict)
1543 Dropped setsum_reindex_id, setprod_reindex_id
1544 (simple variants of setsum.reindex [symmetric], setprod.reindex [symmetric]).
1548 * Abolished slightly odd global lattice interpretation for min/max.
1550 Fact consolidations:
1551 min_max.inf_assoc ~> min.assoc
1552 min_max.inf_commute ~> min.commute
1553 min_max.inf_left_commute ~> min.left_commute
1554 min_max.inf_idem ~> min.idem
1555 min_max.inf_left_idem ~> min.left_idem
1556 min_max.inf_right_idem ~> min.right_idem
1557 min_max.sup_assoc ~> max.assoc
1558 min_max.sup_commute ~> max.commute
1559 min_max.sup_left_commute ~> max.left_commute
1560 min_max.sup_idem ~> max.idem
1561 min_max.sup_left_idem ~> max.left_idem
1562 min_max.sup_inf_distrib1 ~> max_min_distrib2
1563 min_max.sup_inf_distrib2 ~> max_min_distrib1
1564 min_max.inf_sup_distrib1 ~> min_max_distrib2
1565 min_max.inf_sup_distrib2 ~> min_max_distrib1
1566 min_max.distrib ~> min_max_distribs
1567 min_max.inf_absorb1 ~> min.absorb1
1568 min_max.inf_absorb2 ~> min.absorb2
1569 min_max.sup_absorb1 ~> max.absorb1
1570 min_max.sup_absorb2 ~> max.absorb2
1571 min_max.le_iff_inf ~> min.absorb_iff1
1572 min_max.le_iff_sup ~> max.absorb_iff2
1573 min_max.inf_le1 ~> min.cobounded1
1574 min_max.inf_le2 ~> min.cobounded2
1575 le_maxI1, min_max.sup_ge1 ~> max.cobounded1
1576 le_maxI2, min_max.sup_ge2 ~> max.cobounded2
1577 min_max.le_infI1 ~> min.coboundedI1
1578 min_max.le_infI2 ~> min.coboundedI2
1579 min_max.le_supI1 ~> max.coboundedI1
1580 min_max.le_supI2 ~> max.coboundedI2
1581 min_max.less_infI1 ~> min.strict_coboundedI1
1582 min_max.less_infI2 ~> min.strict_coboundedI2
1583 min_max.less_supI1 ~> max.strict_coboundedI1
1584 min_max.less_supI2 ~> max.strict_coboundedI2
1585 min_max.inf_mono ~> min.mono
1586 min_max.sup_mono ~> max.mono
1587 min_max.le_infI, min_max.inf_greatest ~> min.boundedI
1588 min_max.le_supI, min_max.sup_least ~> max.boundedI
1589 min_max.le_inf_iff ~> min.bounded_iff
1590 min_max.le_sup_iff ~> max.bounded_iff
1592 For min_max.inf_sup_aci, prefer (one of) min.commute, min.assoc,
1593 min.left_commute, min.left_idem, max.commute, max.assoc,
1594 max.left_commute, max.left_idem directly.
1596 For min_max.inf_sup_ord, prefer (one of) min.cobounded1,
1597 min.cobounded2, max.cobounded1m max.cobounded2 directly.
1599 For min_ac or max_ac, prefer more general collection ac_simps.
1603 * Theorem disambiguation Inf_le_Sup (on finite sets) ~>
1604 Inf_fin_le_Sup_fin. INCOMPATIBILITY.
1606 * Qualified constant names Wellfounded.acc, Wellfounded.accp.
1609 * Fact generalization and consolidation:
1610 neq_one_mod_two, mod_2_not_eq_zero_eq_one_int ~> not_mod_2_eq_0_eq_1
1614 * Purely algebraic definition of even. Fact generalization and
1616 nat_even_iff_2_dvd, int_even_iff_2_dvd ~> even_iff_2_dvd
1617 even_zero_(nat|int) ~> even_zero
1621 * Abolished neg_numeral.
1622 - Canonical representation for minus one is "- 1".
1623 - Canonical representation for other negative numbers is "- (numeral _)".
1624 - When devising rule sets for number calculation, consider the
1625 following canonical cases: 0, 1, numeral _, - 1, - numeral _.
1626 - HOLogic.dest_number also recognizes numerals in non-canonical forms
1627 like "numeral One", "- numeral One", "- 0" and even "- ... - _".
1628 - Syntax for negative numerals is mere input syntax.
1632 * Reduced name variants for rules on associativity and commutativity:
1634 add_assoc ~> add.assoc
1635 add_commute ~> add.commute
1636 add_left_commute ~> add.left_commute
1637 mult_assoc ~> mult.assoc
1638 mult_commute ~> mult.commute
1639 mult_left_commute ~> mult.left_commute
1640 nat_add_assoc ~> add.assoc
1641 nat_add_commute ~> add.commute
1642 nat_add_left_commute ~> add.left_commute
1643 nat_mult_assoc ~> mult.assoc
1644 nat_mult_commute ~> mult.commute
1645 eq_assoc ~> iff_assoc
1646 eq_left_commute ~> iff_left_commute
1650 * Fact collections add_ac and mult_ac are considered old-fashioned.
1651 Prefer ac_simps instead, or specify rules
1652 (add|mult).(assoc|commute|left_commute) individually.
1654 * Elimination of fact duplicates:
1655 equals_zero_I ~> minus_unique
1656 diff_eq_0_iff_eq ~> right_minus_eq
1657 nat_infinite ~> infinite_UNIV_nat
1658 int_infinite ~> infinite_UNIV_int
1662 * Fact name consolidation:
1663 diff_def, diff_minus, ab_diff_minus ~> diff_conv_add_uminus
1664 minus_le_self_iff ~> neg_less_eq_nonneg
1665 le_minus_self_iff ~> less_eq_neg_nonpos
1666 neg_less_nonneg ~> neg_less_pos
1667 less_minus_self_iff ~> less_neg_neg [simp]
1671 * More simplification rules on unary and binary minus:
1672 add_diff_cancel, add_diff_cancel_left, add_le_same_cancel1,
1673 add_le_same_cancel2, add_less_same_cancel1, add_less_same_cancel2,
1674 add_minus_cancel, diff_add_cancel, le_add_same_cancel1,
1675 le_add_same_cancel2, less_add_same_cancel1, less_add_same_cancel2,
1676 minus_add_cancel, uminus_add_conv_diff. These correspondingly have
1677 been taken away from fact collections algebra_simps and field_simps.
1680 To restore proofs, the following patterns are helpful:
1682 a) Arbitrary failing proof not involving "diff_def":
1683 Consider simplification with algebra_simps or field_simps.
1685 b) Lifting rules from addition to subtraction:
1686 Try with "using <rule for addition> of [... "- _" ...]" by simp".
1688 c) Simplification with "diff_def": just drop "diff_def".
1689 Consider simplification with algebra_simps or field_simps;
1690 or the brute way with
1691 "simp add: diff_conv_add_uminus del: add_uminus_conv_diff".
1693 * Introduce bdd_above and bdd_below in theory
1694 Conditionally_Complete_Lattices, use them instead of explicitly
1695 stating boundedness of sets.
1697 * ccpo.admissible quantifies only over non-empty chains to allow more
1698 syntax-directed proof rules; the case of the empty chain shows up as
1699 additional case in fixpoint induction proofs. INCOMPATIBILITY.
1701 * Removed and renamed theorems in Series:
1702 summable_le ~> suminf_le
1703 suminf_le ~> suminf_le_const
1704 series_pos_le ~> setsum_le_suminf
1705 series_pos_less ~> setsum_less_suminf
1706 suminf_ge_zero ~> suminf_nonneg
1707 suminf_gt_zero ~> suminf_pos
1708 suminf_gt_zero_iff ~> suminf_pos_iff
1709 summable_sumr_LIMSEQ_suminf ~> summable_LIMSEQ
1710 suminf_0_le ~> suminf_nonneg [rotate]
1711 pos_summable ~> summableI_nonneg_bounded
1712 ratio_test ~> summable_ratio_test
1714 removed series_zero, replaced by sums_finite
1716 removed auxiliary lemmas:
1718 sumr_offset, sumr_offset2, sumr_offset3, sumr_offset4, sumr_group,
1719 half, le_Suc_ex_iff, lemma_realpow_diff_sumr,
1720 real_setsum_nat_ivl_bounded, summable_le2, ratio_test_lemma2,
1721 sumr_minus_one_realpow_zerom, sumr_one_lb_realpow_zero,
1722 summable_convergent_sumr_iff, sumr_diff_mult_const
1726 * Replace (F)DERIV syntax by has_derivative:
1727 - "(f has_derivative f') (at x within s)" replaces "FDERIV f x : s : f'"
1729 - "(f has_field_derivative f') (at x within s)" replaces "DERIV f x : s : f'"
1731 - "f differentiable at x within s" replaces "_ differentiable _ in _" syntax
1733 - removed constant isDiff
1735 - "DERIV f x : f'" and "FDERIV f x : f'" syntax is only available as
1738 - "DERIV f x : s : f'" and "FDERIV f x : s : f'" syntax removed.
1740 - Renamed FDERIV_... lemmas to has_derivative_...
1742 - renamed deriv (the syntax constant used for "DERIV _ _ :> _") to DERIV
1744 - removed DERIV_intros, has_derivative_eq_intros
1746 - introduced derivative_intros and deriative_eq_intros which
1747 includes now rules for DERIV, has_derivative and
1748 has_vector_derivative.
1751 differentiable_def ~> real_differentiable_def
1752 differentiableE ~> real_differentiableE
1753 fderiv_def ~> has_derivative_at
1754 field_fderiv_def ~> field_has_derivative_at
1755 isDiff_der ~> differentiable_def
1756 deriv_fderiv ~> has_field_derivative_def
1757 deriv_def ~> DERIV_def
1761 * Include more theorems in continuous_intros. Remove the
1762 continuous_on_intros, isCont_intros collections, these facts are now
1763 in continuous_intros.
1765 * Theorems about complex numbers are now stated only using Re and Im,
1766 the Complex constructor is not used anymore. It is possible to use
1767 primcorec to defined the behaviour of a complex-valued function.
1769 Removed theorems about the Complex constructor from the simpset, they
1770 are available as the lemma collection legacy_Complex_simps. This
1773 i_complex_of_real: "ii * complex_of_real r = Complex 0 r".
1775 Instead the reverse direction is supported with
1776 Complex_eq: "Complex a b = a + \<i> * b"
1778 Moved csqrt from Fundamental_Algebra_Theorem to Complex.
1781 Re/Im ~> complex.sel
1782 complex_Re/Im_zero ~> zero_complex.sel
1783 complex_Re/Im_add ~> plus_complex.sel
1784 complex_Re/Im_minus ~> uminus_complex.sel
1785 complex_Re/Im_diff ~> minus_complex.sel
1786 complex_Re/Im_one ~> one_complex.sel
1787 complex_Re/Im_mult ~> times_complex.sel
1788 complex_Re/Im_inverse ~> inverse_complex.sel
1789 complex_Re/Im_scaleR ~> scaleR_complex.sel
1790 complex_Re/Im_i ~> ii.sel
1791 complex_Re/Im_cnj ~> cnj.sel
1792 Re/Im_cis ~> cis.sel
1794 complex_divide_def ~> divide_complex_def
1795 complex_norm_def ~> norm_complex_def
1796 cmod_def ~> norm_complex_de
1810 * Theory Lubs moved HOL image to HOL-Library. It is replaced by
1811 Conditionally_Complete_Lattices. INCOMPATIBILITY.
1813 * HOL-Library: new theory src/HOL/Library/Tree.thy.
1815 * HOL-Library: removed theory src/HOL/Library/Kleene_Algebra.thy; it
1816 is subsumed by session Kleene_Algebra in AFP.
1818 * HOL-Library / theory RBT: various constants and facts are hidden;
1819 lifting setup is unregistered. INCOMPATIBILITY.
1821 * HOL-Cardinals: new theory src/HOL/Cardinals/Ordinal_Arithmetic.thy.
1823 * HOL-Word: bit representations prefer type bool over type bit.
1827 - Abandoned fact collection "word_arith_alts", which is a duplicate
1828 of "word_arith_wis".
1829 - Dropped first (duplicated) element in fact collections
1830 "sint_word_ariths", "word_arith_alts", "uint_word_ariths",
1831 "uint_word_arith_bintrs".
1833 * HOL-Number_Theory:
1834 - consolidated the proofs of the binomial theorem
1835 - the function fib is again of type nat => nat and not overloaded
1836 - no more references to Old_Number_Theory in the HOL libraries
1841 * HOL-Multivariate_Analysis:
1842 - Type class ordered_real_vector for ordered vector spaces.
1843 - New theory Complex_Basic_Analysis defining complex derivatives,
1844 holomorphic functions, etc., ported from HOL Light's canal.ml.
1845 - Changed order of ordered_euclidean_space to be compatible with
1846 pointwise ordering on products. Therefore instance of
1847 conditionally_complete_lattice and ordered_real_vector.
1848 INCOMPATIBILITY: use box instead of greaterThanLessThan or
1849 explicit set-comprehensions with eucl_less for other (half-)open
1851 - removed dependencies on type class ordered_euclidean_space with
1852 introduction of "cbox" on euclidean_space
1855 mem_interval ~> mem_box
1856 interval_eq_empty ~> box_eq_empty
1857 interval_ne_empty ~> box_ne_empty
1858 interval_sing(1) ~> cbox_sing
1859 interval_sing(2) ~> box_sing
1860 subset_interval_imp ~> subset_box_imp
1861 subset_interval ~> subset_box
1862 open_interval ~> open_box
1863 closed_interval ~> closed_cbox
1864 interior_closed_interval ~> interior_cbox
1865 bounded_closed_interval ~> bounded_cbox
1866 compact_interval ~> compact_cbox
1867 bounded_subset_closed_interval_symmetric ~> bounded_subset_cbox_symmetric
1868 bounded_subset_closed_interval ~> bounded_subset_cbox
1869 mem_interval_componentwiseI ~> mem_box_componentwiseI
1870 convex_box ~> convex_prod
1871 rel_interior_real_interval ~> rel_interior_real_box
1872 convex_interval ~> convex_box
1873 convex_hull_eq_real_interval ~> convex_hull_eq_real_cbox
1874 frechet_derivative_within_closed_interval ~> frechet_derivative_within_cbox
1875 content_closed_interval' ~> content_cbox'
1876 elementary_subset_interval ~> elementary_subset_box
1877 diameter_closed_interval ~> diameter_cbox
1878 frontier_closed_interval ~> frontier_cbox
1879 frontier_open_interval ~> frontier_box
1880 bounded_subset_open_interval_symmetric ~> bounded_subset_box_symmetric
1881 closure_open_interval ~> closure_box
1882 open_closed_interval_convex ~> open_cbox_convex
1883 open_interval_midpoint ~> box_midpoint
1884 content_image_affinity_interval ~> content_image_affinity_cbox
1885 is_interval_interval ~> is_interval_cbox + is_interval_box + is_interval_closed_interval
1886 bounded_interval ~> bounded_closed_interval + bounded_boxes
1888 - respective theorems for intervals over the reals:
1889 content_closed_interval + content_cbox
1890 has_integral + has_integral_real
1891 fine_division_exists + fine_division_exists_real
1892 has_integral_null + has_integral_null_real
1893 tagged_division_union_interval + tagged_division_union_interval_real
1894 has_integral_const + has_integral_const_real
1895 integral_const + integral_const_real
1896 has_integral_bound + has_integral_bound_real
1897 integrable_continuous + integrable_continuous_real
1898 integrable_subinterval + integrable_subinterval_real
1899 has_integral_reflect_lemma + has_integral_reflect_lemma_real
1900 integrable_reflect + integrable_reflect_real
1901 integral_reflect + integral_reflect_real
1902 image_affinity_interval + image_affinity_cbox
1903 image_smult_interval + image_smult_cbox
1904 integrable_const + integrable_const_ivl
1905 integrable_on_subinterval + integrable_on_subcbox
1908 derivative_linear ~> has_derivative_bounded_linear
1909 derivative_is_linear ~> has_derivative_linear
1910 bounded_linear_imp_linear ~> bounded_linear.linear
1913 - Renamed positive_integral to nn_integral:
1915 . Renamed all lemmas "*positive_integral*" to *nn_integral*"
1916 positive_integral_positive ~> nn_integral_nonneg
1918 . Renamed abbreviation integral\<^sup>P to integral\<^sup>N.
1920 - replaced the Lebesgue integral on real numbers by the more general
1921 Bochner integral for functions into a real-normed vector space.
1923 integral_zero ~> integral_zero / integrable_zero
1924 integral_minus ~> integral_minus / integrable_minus
1925 integral_add ~> integral_add / integrable_add
1926 integral_diff ~> integral_diff / integrable_diff
1927 integral_setsum ~> integral_setsum / integrable_setsum
1928 integral_multc ~> integral_mult_left / integrable_mult_left
1929 integral_cmult ~> integral_mult_right / integrable_mult_right
1930 integral_triangle_inequality~> integral_norm_bound
1931 integrable_nonneg ~> integrableI_nonneg
1932 integral_positive ~> integral_nonneg_AE
1933 integrable_abs_iff ~> integrable_abs_cancel
1934 positive_integral_lim_INF ~> nn_integral_liminf
1935 lebesgue_real_affine ~> lborel_real_affine
1936 borel_integral_has_integral ~> has_integral_lebesgue_integral
1937 integral_indicator ~>
1938 integral_real_indicator / integrable_real_indicator
1939 positive_integral_fst ~> nn_integral_fst'
1940 positive_integral_fst_measurable ~> nn_integral_fst
1941 positive_integral_snd_measurable ~> nn_integral_snd
1943 integrable_fst_measurable ~>
1944 integral_fst / integrable_fst / AE_integrable_fst
1946 integrable_snd_measurable ~>
1947 integral_snd / integrable_snd / AE_integrable_snd
1949 integral_monotone_convergence ~>
1950 integral_monotone_convergence / integrable_monotone_convergence
1952 integral_monotone_convergence_at_top ~>
1953 integral_monotone_convergence_at_top /
1954 integrable_monotone_convergence_at_top
1956 has_integral_iff_positive_integral_lebesgue ~>
1957 has_integral_iff_has_bochner_integral_lebesgue_nonneg
1959 lebesgue_integral_has_integral ~>
1960 has_integral_integrable_lebesgue_nonneg
1962 positive_integral_lebesgue_has_integral ~>
1963 integral_has_integral_lebesgue_nonneg /
1964 integrable_has_integral_lebesgue_nonneg
1966 lebesgue_integral_real_affine ~>
1967 nn_integral_real_affine
1969 has_integral_iff_positive_integral_lborel ~>
1970 integral_has_integral_nonneg / integrable_has_integral_nonneg
1972 The following theorems where removed:
1974 lebesgue_integral_nonneg
1975 lebesgue_integral_uminus
1976 lebesgue_integral_cmult
1977 lebesgue_integral_multc
1978 lebesgue_integral_cmult_nonneg
1979 integral_cmul_indicator
1982 - Formalized properties about exponentially, Erlang, and normal
1983 distributed random variables.
1985 * HOL-Decision_Procs: Separate command 'approximate' for approximative
1986 computation in src/HOL/Decision_Procs/Approximation. Minor
1992 * The signature and semantics of Document.Snapshot.cumulate_markup /
1993 select_markup have been clarified. Markup is now traversed in the
1994 order of reports given by the prover: later markup is usually more
1995 specific and may override results accumulated so far. The elements
1996 guard is mandatory and checked precisely. Subtle INCOMPATIBILITY.
1998 * Substantial reworking of internal PIDE protocol communication
1999 channels. INCOMPATIBILITY.
2004 * Subtle change of semantics of Thm.eq_thm: theory stamps are not
2005 compared (according to Thm.thm_ord), but assumed to be covered by the
2006 current background theory. Thus equivalent data produced in different
2007 branches of the theory graph usually coincides (e.g. relevant for
2008 theory merge). Note that the softer Thm.eq_thm_prop is often more
2009 appropriate than Thm.eq_thm.
2011 * Proper context for basic Simplifier operations: rewrite_rule,
2012 rewrite_goals_rule, rewrite_goals_tac etc. INCOMPATIBILITY, need to
2013 pass runtime Proof.context (and ensure that the simplified entity
2014 actually belongs to it).
2016 * Proper context discipline for read_instantiate and instantiate_tac:
2017 variables that are meant to become schematic need to be given as
2018 fixed, and are generalized by the explicit context of local variables.
2019 This corresponds to Isar attributes "where" and "of" with 'for'
2020 declaration. INCOMPATIBILITY, also due to potential change of indices
2021 of schematic variables.
2023 * Moved ML_Compiler.exn_trace and other operations on exceptions to
2024 structure Runtime. Minor INCOMPATIBILITY.
2026 * Discontinued old Toplevel.debug in favour of system option
2027 "ML_exception_trace", which may be also declared within the context
2028 via "declare [[ML_exception_trace = true]]". Minor INCOMPATIBILITY.
2030 * Renamed configuration option "ML_trace" to "ML_source_trace". Minor
2033 * Configuration option "ML_print_depth" controls the pretty-printing
2034 depth of the ML compiler within the context. The old print_depth in
2035 ML is still available as default_print_depth, but rarely used. Minor
2038 * Toplevel function "use" refers to raw ML bootstrap environment,
2039 without Isar context nor antiquotations. Potential INCOMPATIBILITY.
2040 Note that 'ML_file' is the canonical command to load ML files into the
2043 * Simplified programming interface to define ML antiquotations, see
2044 structure ML_Antiquotation. Minor INCOMPATIBILITY.
2046 * ML antiquotation @{here} refers to its source position, which is
2047 occasionally useful for experimentation and diagnostic purposes.
2049 * ML antiquotation @{path} produces a Path.T value, similarly to
2050 Path.explode, but with compile-time check against the file-system and
2051 some PIDE markup. Note that unlike theory source, ML does not have a
2052 well-defined master directory, so an absolute symbolic path
2053 specification is usually required, e.g. "~~/src/HOL".
2055 * ML antiquotation @{print} inlines a function to print an arbitrary
2056 ML value, which is occasionally useful for diagnostic or demonstration
2062 * Proof General with its traditional helper scripts is now an optional
2063 Isabelle component, e.g. see ProofGeneral-4.2-2 from the Isabelle
2064 component repository http://isabelle.in.tum.de/components/. Note that
2065 the "system" manual provides general explanations about add-on
2066 components, especially those that are not bundled with the release.
2068 * The raw Isabelle process executable has been renamed from
2069 "isabelle-process" to "isabelle_process", which conforms to common
2070 shell naming conventions, and allows to define a shell function within
2071 the Isabelle environment to avoid dynamic path lookup. Rare
2072 incompatibility for old tools that do not use the ISABELLE_PROCESS
2075 * Former "isabelle tty" has been superseded by "isabelle console",
2076 with implicit build like "isabelle jedit", and without the mostly
2077 obsolete Isar TTY loop.
2079 * Simplified "isabelle display" tool. Settings variables DVI_VIEWER
2080 and PDF_VIEWER now refer to the actual programs, not shell
2081 command-lines. Discontinued option -c: invocation may be asynchronous
2082 via desktop environment, without any special precautions. Potential
2083 INCOMPATIBILITY with ambitious private settings.
2085 * Removed obsolete "isabelle unsymbolize". Note that the usual format
2086 for email communication is the Unicode rendering of Isabelle symbols,
2087 as produced by Isabelle/jEdit, for example.
2089 * Removed obsolete tool "wwwfind". Similar functionality may be
2090 integrated into Isabelle/jEdit eventually.
2092 * Improved 'display_drafts' concerning desktop integration and
2093 repeated invocation in PIDE front-end: re-use single file
2094 $ISABELLE_HOME_USER/tmp/drafts.pdf and corresponding views.
2096 * Session ROOT specifications require explicit 'document_files' for
2097 robust dependencies on LaTeX sources. Only these explicitly given
2098 files are copied to the document output directory, before document
2099 processing is started.
2101 * Windows: support for regular TeX installation (e.g. MiKTeX) instead
2102 of TeX Live from Cygwin.
2106 New in Isabelle2013-2 (December 2013)
2107 -------------------------------------
2109 *** Prover IDE -- Isabelle/Scala/jEdit ***
2111 * More robust editing of running commands with internal forks,
2112 e.g. non-terminating 'by' steps.
2114 * More relaxed Sledgehammer panel: avoid repeated application of query
2115 after edits surrounding the command location.
2117 * More status information about commands that are interrupted
2118 accidentally (via physical event or Poly/ML runtime system signal,
2119 e.g. out-of-memory).
2124 * More robust termination of external processes managed by
2125 Isabelle/ML: support cancellation of tasks within the range of
2126 milliseconds, as required for PIDE document editing with automatically
2127 tried tools (e.g. Sledgehammer).
2129 * Reactivated Isabelle/Scala kill command for external processes on
2130 Mac OS X, which was accidentally broken in Isabelle2013-1 due to a
2131 workaround for some Debian/Ubuntu Linux versions from 2013.
2135 New in Isabelle2013-1 (November 2013)
2136 -------------------------------------
2140 * Discontinued obsolete 'uses' within theory header. Note that
2141 commands like 'ML_file' work without separate declaration of file
2142 dependencies. Minor INCOMPATIBILITY.
2144 * Discontinued redundant 'use' command, which was superseded by
2145 'ML_file' in Isabelle2013. Minor INCOMPATIBILITY.
2147 * Simplified subscripts within identifiers, using plain \<^sub>
2148 instead of the second copy \<^isub> and \<^isup>. Superscripts are
2149 only for literal tokens within notation; explicit mixfix annotations
2150 for consts or fixed variables may be used as fall-back for unusual
2151 names. Obsolete \<twosuperior> has been expanded to \<^sup>2 in
2152 Isabelle/HOL. INCOMPATIBILITY, use "isabelle update_sub_sup" to
2153 standardize symbols as a starting point for further manual cleanup.
2154 The ML reference variable "legacy_isub_isup" may be set as temporary
2155 workaround, to make the prover accept a subset of the old identifier
2158 * Document antiquotations: term style "isub" has been renamed to
2159 "sub". Minor INCOMPATIBILITY.
2161 * Uniform management of "quick_and_dirty" as system option (see also
2162 "isabelle options"), configuration option within the context (see also
2163 Config.get in Isabelle/ML), and attribute in Isabelle/Isar. Minor
2164 INCOMPATIBILITY, need to use more official Isabelle means to access
2165 quick_and_dirty, instead of historical poking into mutable reference.
2167 * Renamed command 'print_configs' to 'print_options'. Minor
2170 * Proper diagnostic command 'print_state'. Old 'pr' (with its
2171 implicit change of some global references) is retained for now as
2172 control command, e.g. for ProofGeneral 3.7.x.
2174 * Discontinued 'print_drafts' command with its old-fashioned PS output
2175 and Unix command-line print spooling. Minor INCOMPATIBILITY: use
2176 'display_drafts' instead and print via the regular document viewer.
2178 * Updated and extended "isar-ref" and "implementation" manual,
2179 eliminated old "ref" manual.
2182 *** Prover IDE -- Isabelle/Scala/jEdit ***
2184 * New manual "jedit" for Isabelle/jEdit, see isabelle doc or
2185 Documentation panel.
2187 * Dockable window "Documentation" provides access to Isabelle
2190 * Dockable window "Find" provides query operations for formal entities
2191 (GUI front-end to 'find_theorems' command).
2193 * Dockable window "Sledgehammer" manages asynchronous / parallel
2194 sledgehammer runs over existing document sources, independently of
2195 normal editing and checking process.
2197 * Dockable window "Timing" provides an overview of relevant command
2198 timing information, depending on option jedit_timing_threshold. The
2199 same timing information is shown in the extended tooltip of the
2200 command keyword, when hovering the mouse over it while the CONTROL or
2201 COMMAND modifier is pressed.
2203 * Improved dockable window "Theories": Continuous checking of proof
2204 document (visible and required parts) may be controlled explicitly,
2205 using check box or shortcut "C+e ENTER". Individual theory nodes may
2206 be marked explicitly as required and checked in full, using check box
2207 or shortcut "C+e SPACE".
2209 * Improved completion mechanism, which is now managed by the
2210 Isabelle/jEdit plugin instead of SideKick. Refined table of Isabelle
2211 symbol abbreviations (see $ISABELLE_HOME/etc/symbols).
2213 * Standard jEdit keyboard shortcut C+b complete-word is remapped to
2214 isabelle.complete for explicit completion in Isabelle sources.
2215 INCOMPATIBILITY wrt. jEdit defaults, may have to invent new shortcuts
2216 to resolve conflict.
2218 * Improved support of various "minor modes" for Isabelle NEWS,
2219 options, session ROOT etc., with completion and SideKick tree view.
2221 * Strictly monotonic document update, without premature cancellation of
2222 running transactions that are still needed: avoid reset/restart of
2223 such command executions while editing.
2225 * Support for asynchronous print functions, as overlay to existing
2228 * Support for automatic tools in HOL, which try to prove or disprove
2229 toplevel theorem statements.
2231 * Action isabelle.reset-font-size resets main text area font size
2232 according to Isabelle/Scala plugin option "jedit_font_reset_size" (see
2233 also "Plugin Options / Isabelle / General"). It can be bound to some
2234 keyboard shortcut by the user (e.g. C+0 and/or C+NUMPAD0).
2236 * File specifications in jEdit (e.g. file browser) may refer to
2237 $ISABELLE_HOME and $ISABELLE_HOME_USER on all platforms. Discontinued
2238 obsolete $ISABELLE_HOME_WINDOWS variable.
2240 * Improved support for Linux look-and-feel "GTK+", see also "Utilities
2241 / Global Options / Appearance".
2243 * Improved support of native Mac OS X functionality via "MacOSX"
2244 plugin, which is now enabled by default.
2249 * Commands 'interpretation' and 'sublocale' are now target-sensitive.
2250 In particular, 'interpretation' allows for non-persistent
2251 interpretation within "context ... begin ... end" blocks offering a
2252 light-weight alternative to 'sublocale'. See "isar-ref" manual for
2255 * Improved locales diagnostic command 'print_dependencies'.
2257 * Discontinued obsolete 'axioms' command, which has been marked as
2258 legacy since Isabelle2009-2. INCOMPATIBILITY, use 'axiomatization'
2259 instead, while observing its uniform scope for polymorphism.
2261 * Discontinued empty name bindings in 'axiomatization'.
2264 * System option "proofs" has been discontinued. Instead the global
2265 state of Proofterm.proofs is persistently compiled into logic images
2266 as required, notably HOL-Proofs. Users no longer need to change
2267 Proofterm.proofs dynamically. Minor INCOMPATIBILITY.
2269 * Syntax translation functions (print_translation etc.) always depend
2270 on Proof.context. Discontinued former "(advanced)" option -- this is
2271 now the default. Minor INCOMPATIBILITY.
2273 * Former global reference trace_unify_fail is now available as
2274 configuration option "unify_trace_failure" (global context only).
2276 * SELECT_GOAL now retains the syntactic context of the overall goal
2277 state (schematic variables etc.). Potential INCOMPATIBILITY in rare
2283 * Stronger precedence of syntax for big intersection and union on
2284 sets, in accordance with corresponding lattice operations.
2287 * Notation "{p:A. P}" now allows tuple patterns as well.
2289 * Nested case expressions are now translated in a separate check phase
2290 rather than during parsing. The data for case combinators is separated
2291 from the datatype package. The declaration attribute
2292 "case_translation" can be used to register new case combinators:
2294 declare [[case_translation case_combinator constructor1 ... constructorN]]
2297 - 'code_printing' unifies 'code_const' / 'code_type' / 'code_class' /
2299 - 'code_identifier' declares name hints for arbitrary identifiers in
2300 generated code, subsuming 'code_modulename'.
2302 See the isar-ref manual for syntax diagrams, and the HOL theories for
2305 * Attibute 'code': 'code' now declares concrete and abstract code
2306 equations uniformly. Use explicit 'code equation' and 'code abstract'
2307 to distinguish both when desired.
2309 * Discontinued theories Code_Integer and Efficient_Nat by a more
2310 fine-grain stack of theories Code_Target_Int, Code_Binary_Nat,
2311 Code_Target_Nat and Code_Target_Numeral. See the tutorial on code
2312 generation for details. INCOMPATIBILITY.
2314 * Numeric types are mapped by default to target language numerals:
2315 natural (replaces former code_numeral) and integer (replaces former
2316 code_int). Conversions are available as integer_of_natural /
2317 natural_of_integer / integer_of_nat / nat_of_integer (in HOL) and
2318 Code_Numeral.integer_of_natural / Code_Numeral.natural_of_integer (in
2319 ML). INCOMPATIBILITY.
2321 * Function package: For mutually recursive functions f and g, separate
2322 cases rules f.cases and g.cases are generated instead of unusable
2323 f_g.cases which exposed internal sum types. Potential INCOMPATIBILITY,
2324 in the case that the unusable rule was used nevertheless.
2326 * Function package: For each function f, new rules f.elims are
2327 generated, which eliminate equalities of the form "f x = t".
2329 * New command 'fun_cases' derives ad-hoc elimination rules for
2330 function equations as simplified instances of f.elims, analogous to
2331 inductive_cases. See ~~/src/HOL/ex/Fundefs.thy for some examples.
2334 - parametrized correspondence relations are now supported:
2335 + parametricity theorems for the raw term can be specified in
2336 the command lift_definition, which allow us to generate stronger
2338 + setup_lifting generates stronger transfer rules if parametric
2339 correspondence relation can be generated
2340 + various new properties of the relator must be specified to support
2342 + parametricity theorem for the Quotient relation can be specified
2343 - setup_lifting generates domain rules for the Transfer package
2344 - stronger reflexivity prover of respectfulness theorems for type
2346 - ===> and --> are now local. The symbols can be introduced
2347 by interpreting the locale lifting_syntax (typically in an
2349 - Lifting/Transfer relevant parts of Library/Quotient_* are now in
2350 Main. Potential INCOMPATIBILITY
2351 - new commands for restoring and deleting Lifting/Transfer context:
2352 lifting_forget, lifting_update
2353 - the command print_quotmaps was renamed to print_quot_maps.
2357 - better support for domains in Transfer: replace Domainp T
2358 by the actual invariant in a transferred goal
2359 - transfer rules can have as assumptions other transfer rules
2360 - Experimental support for transferring from the raw level to the
2361 abstract level: Transfer.transferred attribute
2362 - Attribute version of the transfer method: untransferred attribute
2364 * Reification and reflection:
2365 - Reification is now directly available in HOL-Main in structure
2367 - Reflection now handles multiple lists with variables also.
2368 - The whole reflection stack has been decomposed into conversions.
2371 * Revised devices for recursive definitions over finite sets:
2372 - Only one fundamental fold combinator on finite set remains:
2373 Finite_Set.fold :: ('a => 'b => 'b) => 'b => 'a set => 'b
2374 This is now identity on infinite sets.
2375 - Locales ("mini packages") for fundamental definitions with
2376 Finite_Set.fold: folding, folding_idem.
2377 - Locales comm_monoid_set, semilattice_order_set and
2378 semilattice_neutr_order_set for big operators on sets.
2379 See theory Big_Operators for canonical examples.
2380 Note that foundational constants comm_monoid_set.F and
2381 semilattice_set.F correspond to former combinators fold_image
2382 and fold1 respectively. These are now gone. You may use
2383 those foundational constants as substitutes, but it is
2384 preferable to interpret the above locales accordingly.
2385 - Dropped class ab_semigroup_idem_mult (special case of lattice,
2386 no longer needed in connection with Finite_Set.fold etc.)
2388 card.union_inter ~> card_Un_Int [symmetric]
2389 card.union_disjoint ~> card_Un_disjoint
2392 * Locale hierarchy for abstract orderings and (semi)lattices.
2394 * Complete_Partial_Order.admissible is defined outside the type class
2395 ccpo, but with mandatory prefix ccpo. Admissibility theorems lose the
2396 class predicate assumption or sort constraint when possible.
2399 * Introduce type class "conditionally_complete_lattice": Like a
2400 complete lattice but does not assume the existence of the top and
2401 bottom elements. Allows to generalize some lemmas about reals and
2402 extended reals. Removed SupInf and replaced it by the instantiation
2403 of conditionally_complete_lattice for real. Renamed lemmas about
2404 conditionally-complete lattice from Sup_... to cSup_... and from
2405 Inf_... to cInf_... to avoid hidding of similar complete lattice
2408 * Introduce type class linear_continuum as combination of
2409 conditionally-complete lattices and inner dense linorders which have
2410 more than one element. INCOMPATIBILITY.
2412 * Introduced type classes order_top and order_bot. The old classes top
2413 and bot only contain the syntax without assumptions. INCOMPATIBILITY:
2414 Rename bot -> order_bot, top -> order_top
2416 * Introduce type classes "no_top" and "no_bot" for orderings without
2417 top and bottom elements.
2419 * Split dense_linorder into inner_dense_order and no_top, no_bot.
2421 * Complex_Main: Unify and move various concepts from
2422 HOL-Multivariate_Analysis to HOL-Complex_Main.
2424 - Introduce type class (lin)order_topology and
2425 linear_continuum_topology. Allows to generalize theorems about
2426 limits and order. Instances are reals and extended reals.
2428 - continuous and continuos_on from Multivariate_Analysis:
2429 "continuous" is the continuity of a function at a filter. "isCont"
2430 is now an abbrevitation: "isCont x f == continuous (at _) f".
2432 Generalized continuity lemmas from isCont to continuous on an
2435 - compact from Multivariate_Analysis. Use Bolzano's lemma to prove
2436 compactness of closed intervals on reals. Continuous functions
2437 attain infimum and supremum on compact sets. The inverse of a
2438 continuous function is continuous, when the function is continuous
2441 - connected from Multivariate_Analysis. Use it to prove the
2442 intermediate value theorem. Show connectedness of intervals on
2443 linear_continuum_topology).
2445 - first_countable_topology from Multivariate_Analysis. Is used to
2446 show equivalence of properties on the neighbourhood filter of x and
2447 on all sequences converging to x.
2449 - FDERIV: Definition of has_derivative moved to Deriv.thy. Moved
2450 theorems from Library/FDERIV.thy to Deriv.thy and base the
2451 definition of DERIV on FDERIV. Add variants of DERIV and FDERIV
2452 which are restricted to sets, i.e. to represent derivatives from
2455 - Removed the within-filter. It is replaced by the principal filter:
2457 F within X = inf F (principal X)
2459 - Introduce "at x within U" as a single constant, "at x" is now an
2460 abbreviation for "at x within UNIV"
2462 - Introduce named theorem collections tendsto_intros,
2463 continuous_intros, continuous_on_intros and FDERIV_intros. Theorems
2464 in tendsto_intros (or FDERIV_intros) are also available as
2465 tendsto_eq_intros (or FDERIV_eq_intros) where the right-hand side
2466 is replaced by a congruence rule. This allows to apply them as
2467 intro rules and then proving equivalence by the simplifier.
2469 - Restructured theories in HOL-Complex_Main:
2471 + Moved RealDef and RComplete into Real
2473 + Introduced Topological_Spaces and moved theorems about
2474 topological spaces, filters, limits and continuity to it
2476 + Renamed RealVector to Real_Vector_Spaces
2478 + Split Lim, SEQ, Series into Topological_Spaces,
2479 Real_Vector_Spaces, and Limits
2481 + Moved Ln and Log to Transcendental
2483 + Moved theorems about continuity from Deriv to Topological_Spaces
2485 - Remove various auxiliary lemmas.
2490 - Added option "spy".
2491 - Reduce incidence of "too high arity" errors.
2495 isar_shrink ~> isar_compress
2497 - Added options "isar_try0", "spy".
2498 - Better support for "isar_proofs".
2499 - MaSh has been fined-tuned and now runs as a local server.
2501 * Improved support for ad hoc overloading of constants (see also
2502 isar-ref manual and ~~/src/HOL/ex/Adhoc_Overloading_Examples.thy).
2504 * Library/Polynomial.thy:
2505 - Use lifting for primitive definitions.
2506 - Explicit conversions from and to lists of coefficients, used for
2508 - Replaced recursion operator poly_rec by fold_coeffs.
2509 - Prefer pre-existing gcd operation for gcd.
2511 poly_eq_iff ~> poly_eq_poly_eq_iff
2512 poly_ext ~> poly_eqI
2513 expand_poly_eq ~> poly_eq_iff
2516 * New Library/Simps_Case_Conv.thy: Provides commands simps_of_case and
2517 case_of_simps to convert function definitions between a list of
2518 equations with patterns on the lhs and a single equation with case
2519 expressions on the rhs. See also Ex/Simps_Case_Conv_Examples.thy.
2521 * New Library/FSet.thy: type of finite sets defined as a subtype of
2522 sets defined by Lifting/Transfer.
2524 * Discontinued theory src/HOL/Library/Eval_Witness. INCOMPATIBILITY.
2526 * Consolidation of library theories on product orders:
2528 Product_Lattice ~> Product_Order -- pointwise order on products
2529 Product_ord ~> Product_Lexorder -- lexicographic order on products
2533 * Imperative-HOL: The MREC combinator is considered legacy and no
2534 longer included by default. INCOMPATIBILITY, use partial_function
2535 instead, or import theory Legacy_Mrec as a fallback.
2537 * HOL-Algebra: Discontinued theories ~~/src/HOL/Algebra/abstract and
2538 ~~/src/HOL/Algebra/poly. Existing theories should be based on
2539 ~~/src/HOL/Library/Polynomial instead. The latter provides
2540 integration with HOL's type classes for rings. INCOMPATIBILITY.
2543 - Various improvements to BNF-based (co)datatype package, including
2544 new commands "primrec_new", "primcorec", and
2545 "datatype_new_compat", as well as documentation. See
2546 "datatypes.pdf" for details.
2547 - New "coinduction" method to avoid some boilerplate (compared to
2550 data ~> datatype_new
2551 codata ~> codatatype
2553 - Renamed many generated theorems, including
2555 map_comp' ~> map_comp
2565 * Spec_Check is a Quickcheck tool for Isabelle/ML. The ML function
2566 "check_property" allows to check specifications of the form "ALL x y
2567 z. prop x y z". See also ~~/src/Tools/Spec_Check/ with its
2568 Examples.thy in particular.
2570 * Improved printing of exception trace in Poly/ML 5.5.1, with regular
2571 tracing output in the command transaction context instead of physical
2572 stdout. See also Toplevel.debug, Toplevel.debugging and
2573 ML_Compiler.exn_trace.
2575 * ML type "theory" is now immutable, without any special treatment of
2576 drafts or linear updates (which could lead to "stale theory" errors in
2577 the past). Discontinued obsolete operations like Theory.copy,
2578 Theory.checkpoint, and the auxiliary type theory_ref. Minor
2581 * More uniform naming of goal functions for skipped proofs:
2583 Skip_Proof.prove ~> Goal.prove_sorry
2584 Skip_Proof.prove_global ~> Goal.prove_sorry_global
2586 Minor INCOMPATIBILITY.
2588 * Simplifier tactics and tools use proper Proof.context instead of
2589 historic type simpset. Old-style declarations like addsimps,
2590 addsimprocs etc. operate directly on Proof.context. Raw type simpset
2591 retains its use as snapshot of the main Simplifier context, using
2592 simpset_of and put_simpset on Proof.context. INCOMPATIBILITY -- port
2593 old tools by making them depend on (ctxt : Proof.context) instead of
2594 (ss : simpset), then turn (simpset_of ctxt) into ctxt.
2596 * Modifiers for classical wrappers (e.g. addWrapper, delWrapper)
2597 operate on Proof.context instead of claset, for uniformity with addIs,
2598 addEs, addDs etc. Note that claset_of and put_claset allow to manage
2599 clasets separately from the context.
2601 * Discontinued obsolete ML antiquotations @{claset} and @{simpset}.
2602 INCOMPATIBILITY, use @{context} instead.
2604 * Antiquotation @{theory_context A} is similar to @{theory A}, but
2605 presents the result as initial Proof.context.
2610 * Discontinued obsolete isabelle usedir, mkdir, make -- superseded by
2611 "isabelle build" in Isabelle2013. INCOMPATIBILITY.
2613 * Discontinued obsolete isabelle-process options -f and -u (former
2614 administrative aliases of option -e). Minor INCOMPATIBILITY.
2616 * Discontinued obsolete isabelle print tool, and PRINT_COMMAND
2619 * Discontinued ISABELLE_DOC_FORMAT settings variable and historic
2620 document formats: dvi.gz, ps, ps.gz -- the default document format is
2623 * Isabelle settings variable ISABELLE_BUILD_JAVA_OPTIONS allows to
2624 specify global resources of the JVM process run by isabelle build.
2626 * Toplevel executable $ISABELLE_HOME/bin/isabelle_scala_script allows
2627 to run Isabelle/Scala source files as standalone programs.
2629 * Improved "isabelle keywords" tool (for old-style ProofGeneral
2630 keyword tables): use Isabelle/Scala operations, which inspect outer
2631 syntax without requiring to build sessions first.
2633 * Sessions may be organized via 'chapter' specifications in the ROOT
2634 file, which determines a two-level hierarchy of browser info. The old
2635 tree-like organization via implicit sub-session relation (with its
2636 tendency towards erratic fluctuation of URLs) has been discontinued.
2637 The default chapter is called "Unsorted". Potential INCOMPATIBILITY
2638 for HTML presentation of theories.
2642 New in Isabelle2013 (February 2013)
2643 -----------------------------------
2647 * Theorem status about oracles and unfinished/failed future proofs is
2648 no longer printed by default, since it is incompatible with
2649 incremental / parallel checking of the persistent document model. ML
2650 function Thm.peek_status may be used to inspect a snapshot of the
2651 ongoing evaluation process. Note that in batch mode --- notably
2652 isabelle build --- the system ensures that future proofs of all
2653 accessible theorems in the theory context are finished (as before).
2655 * Configuration option show_markup controls direct inlining of markup
2656 into the printed representation of formal entities --- notably type
2657 and sort constraints. This enables Prover IDE users to retrieve that
2658 information via tooltips in the output window, for example.
2660 * Command 'ML_file' evaluates ML text from a file directly within the
2661 theory, without any predeclaration via 'uses' in the theory header.
2663 * Old command 'use' command and corresponding keyword 'uses' in the
2664 theory header are legacy features and will be discontinued soon.
2665 Tools that load their additional source files may imitate the
2666 'ML_file' implementation, such that the system can take care of
2667 dependencies properly.
2669 * Discontinued obsolete method fastsimp / tactic fast_simp_tac, which
2670 is called fastforce / fast_force_tac already since Isabelle2011-1.
2672 * Updated and extended "isar-ref" and "implementation" manual, reduced
2673 remaining material in old "ref" manual.
2675 * Improved support for auxiliary contexts that indicate block structure
2676 for specifications. Nesting of "context fixes ... context assumes ..."
2677 and "class ... context ...".
2679 * Attribute "consumes" allows a negative value as well, which is
2680 interpreted relatively to the total number of premises of the rule in
2681 the target context. This form of declaration is stable when exported
2682 from a nested 'context' with additional assumptions. It is the
2683 preferred form for definitional packages, notably cases/rules produced
2684 in HOL/inductive and HOL/function.
2686 * More informative error messages for Isar proof commands involving
2687 lazy enumerations (method applications etc.).
2689 * Refined 'help' command to retrieve outer syntax commands according
2690 to name patterns (with clickable results).
2693 *** Prover IDE -- Isabelle/Scala/jEdit ***
2695 * Parallel terminal proofs ('by') are enabled by default, likewise
2696 proofs that are built into packages like 'datatype', 'function'. This
2697 allows to "run ahead" checking the theory specifications on the
2698 surface, while the prover is still crunching on internal
2699 justifications. Unfinished / cancelled proofs are restarted as
2700 required to complete full proof checking eventually.
2702 * Improved output panel with tooltips, hyperlinks etc. based on the
2703 same Rich_Text_Area as regular Isabelle/jEdit buffers. Activation of
2704 tooltips leads to some window that supports the same recursively,
2705 which can lead to stacks of tooltips as the semantic document content
2706 is explored. ESCAPE closes the whole stack, individual windows may be
2707 closed separately, or detached to become independent jEdit dockables.
2709 * Improved support for commands that produce graph output: the text
2710 message contains a clickable area to open a new instance of the graph
2713 * More robust incremental parsing of outer syntax (partial comments,
2714 malformed symbols). Changing the balance of open/close quotes and
2715 comment delimiters works more conveniently with unfinished situations
2716 that frequently occur in user interaction.
2718 * More efficient painting and improved reactivity when editing large
2719 files. More scalable management of formal document content.
2721 * Smarter handling of tracing messages: prover process pauses after
2722 certain number of messages per command transaction, with some user
2723 dialog to stop or continue. This avoids swamping the front-end with
2724 potentially infinite message streams.
2726 * More plugin options and preferences, based on Isabelle/Scala. The
2727 jEdit plugin option panel provides access to some Isabelle/Scala
2728 options, including tuning parameters for editor reactivity and color
2731 * Dockable window "Symbols" provides some editing support for Isabelle
2734 * Dockable window "Monitor" shows ML runtime statistics. Note that
2735 continuous display of the chart slows down the system.
2737 * Improved editing support for control styles: subscript, superscript,
2738 bold, reset of style -- operating on single symbols or text
2739 selections. Cf. keyboard shortcuts C+e DOWN/UP/RIGHT/LEFT.
2741 * Actions isabelle.increase-font-size and isabelle.decrease-font-size
2742 adjust the main text area font size, and its derivatives for output,
2743 tooltips etc. Cf. keyboard shortcuts C-PLUS and C-MINUS, which often
2744 need to be adapted to local keyboard layouts.
2746 * More reactive completion popup by default: use \t (TAB) instead of
2747 \n (NEWLINE) to minimize intrusion into regular flow of editing. See
2748 also "Plugin Options / SideKick / General / Code Completion Options".
2750 * Implicit check and build dialog of the specified logic session
2751 image. For example, HOL, HOLCF, HOL-Nominal can be produced on
2752 demand, without bundling big platform-dependent heap images in the
2753 Isabelle distribution.
2755 * Uniform Java 7 platform on Linux, Mac OS X, Windows: recent updates
2756 from Oracle provide better multi-platform experience. This version is
2757 now bundled exclusively with Isabelle.
2762 * Code generation for Haskell: restrict unqualified imports from
2763 Haskell Prelude to a small set of fundamental operations.
2765 * Command 'export_code': relative file names are interpreted
2766 relatively to master directory of current theory rather than the
2767 rather arbitrary current working directory. INCOMPATIBILITY.
2769 * Discontinued obsolete attribute "COMP". Potential INCOMPATIBILITY,
2770 use regular rule composition via "OF" / "THEN", or explicit proof
2771 structure instead. Note that Isabelle/ML provides a variety of
2772 operators like COMP, INCR_COMP, COMP_INCR, which need to be applied
2773 with some care where this is really required.
2775 * Command 'typ' supports an additional variant with explicit sort
2776 constraint, to infer and check the most general type conforming to a
2777 given sort. Example (in HOL):
2779 typ "_ * _ * bool * unit" :: finite
2781 * Command 'locale_deps' visualizes all locales and their relations as
2789 - Added MaSh relevance filter based on machine-learning; see the
2790 Sledgehammer manual for details.
2791 - Polished Isar proofs generated with "isar_proofs" option.
2792 - Rationalized type encodings ("type_enc" option).
2793 - Renamed "kill_provers" subcommand to "kill_all".
2795 isar_proof ~> isar_proofs
2796 isar_shrink_factor ~> isar_shrink
2797 max_relevant ~> max_facts
2798 relevance_thresholds ~> fact_thresholds
2800 * Quickcheck: added an optimisation for equality premises. It is
2801 switched on by default, and can be switched off by setting the
2802 configuration quickcheck_optimise_equality to false.
2804 * Quotient: only one quotient can be defined by quotient_type
2808 - generation of an abstraction function equation in lift_definition
2809 - quot_del attribute
2810 - renamed no_abs_code -> no_code (INCOMPATIBILITY.)
2812 * Simproc "finite_Collect" rewrites set comprehensions into pointfree
2815 * Preprocessing of the code generator rewrites set comprehensions into
2816 pointfree expressions.
2818 * The SMT solver Z3 has now by default a restricted set of directly
2819 supported features. For the full set of features (div/mod, nonlinear
2820 arithmetic, datatypes/records) with potential proof reconstruction
2821 failures, enable the configuration option "z3_with_extensions". Minor
2824 * Simplified 'typedef' specifications: historical options for implicit
2825 set definition and alternative name have been discontinued. The
2826 former behavior of "typedef (open) t = A" is now the default, but
2827 written just "typedef t = A". INCOMPATIBILITY, need to adapt theories
2830 * Removed constant "chars"; prefer "Enum.enum" on type "char"
2831 directly. INCOMPATIBILITY.
2833 * Moved operation product, sublists and n_lists from theory Enum to
2834 List. INCOMPATIBILITY.
2836 * Theorem UN_o generalized to SUP_comp. INCOMPATIBILITY.
2838 * Class "comm_monoid_diff" formalises properties of bounded
2839 subtraction, with natural numbers and multisets as typical instances.
2841 * Added combinator "Option.these" with type "'a option set => 'a set".
2843 * Theory "Transitive_Closure": renamed lemmas
2845 reflcl_tranclp -> reflclp_tranclp
2846 rtranclp_reflcl -> rtranclp_reflclp
2850 * Theory "Rings": renamed lemmas (in class semiring)
2852 left_distrib ~> distrib_right
2853 right_distrib ~> distrib_left
2857 * Generalized the definition of limits:
2859 - Introduced the predicate filterlim (LIM x F. f x :> G) which
2860 expresses that when the input values x converge to F then the
2861 output f x converges to G.
2863 - Added filters for convergence to positive (at_top) and negative
2866 - Moved infinity in the norm (at_infinity) from
2867 Multivariate_Analysis to Complex_Main.
2869 - Removed real_tendsto_inf, it is superseded by "LIM x F. f x :>
2874 * Theory "Library/Option_ord" provides instantiation of option type to
2875 lattice type classes.
2877 * Theory "Library/Multiset": renamed
2879 constant fold_mset ~> Multiset.fold
2880 fact fold_mset_commute ~> fold_mset_comm
2884 * Renamed theory Library/List_Prefix to Library/Sublist, with related
2887 - Renamed constants (and related lemmas)
2890 strict_prefix ~> prefix
2892 - Replaced constant "postfix" by "suffixeq" with swapped argument
2893 order (i.e., "postfix xs ys" is now "suffixeq ys xs") and dropped
2894 old infix syntax "xs >>= ys"; use "suffixeq ys xs" instead.
2895 Renamed lemmas accordingly.
2897 - Added constant "list_hembeq" for homeomorphic embedding on
2898 lists. Added abbreviation "sublisteq" for special case
2899 "list_hembeq (op =)".
2901 - Theory Library/Sublist no longer provides "order" and "bot" type
2902 class instances for the prefix order (merely corresponding locale
2903 interpretations). The type class instances are now in theory
2904 Library/Prefix_Order.
2906 - The sublist relation of theory Library/Sublist_Order is now based
2907 on "Sublist.sublisteq". Renamed lemmas accordingly:
2909 le_list_append_le_same_iff ~> Sublist.sublisteq_append_le_same_iff
2910 le_list_append_mono ~> Sublist.list_hembeq_append_mono
2911 le_list_below_empty ~> Sublist.list_hembeq_Nil, Sublist.list_hembeq_Nil2
2912 le_list_Cons_EX ~> Sublist.list_hembeq_ConsD
2913 le_list_drop_Cons2 ~> Sublist.sublisteq_Cons2'
2914 le_list_drop_Cons_neq ~> Sublist.sublisteq_Cons2_neq
2915 le_list_drop_Cons ~> Sublist.sublisteq_Cons'
2916 le_list_drop_many ~> Sublist.sublisteq_drop_many
2917 le_list_filter_left ~> Sublist.sublisteq_filter_left
2918 le_list_rev_drop_many ~> Sublist.sublisteq_rev_drop_many
2919 le_list_rev_take_iff ~> Sublist.sublisteq_append
2920 le_list_same_length ~> Sublist.sublisteq_same_length
2921 le_list_take_many_iff ~> Sublist.sublisteq_append'
2922 less_eq_list.drop ~> less_eq_list_drop
2923 less_eq_list.induct ~> less_eq_list_induct
2924 not_le_list_length ~> Sublist.not_sublisteq_length
2928 * New theory Library/Countable_Set.
2930 * Theory Library/Debug and Library/Parallel provide debugging and
2931 parallel execution for code generated towards Isabelle/ML.
2933 * Theory Library/FuncSet: Extended support for Pi and extensional and
2934 introduce the extensional dependent function space "PiE". Replaced
2935 extensional_funcset by an abbreviation, and renamed lemmas from
2936 extensional_funcset to PiE as follows:
2938 extensional_empty ~> PiE_empty
2939 extensional_funcset_empty_domain ~> PiE_empty_domain
2940 extensional_funcset_empty_range ~> PiE_empty_range
2941 extensional_funcset_arb ~> PiE_arb
2942 extensional_funcset_mem ~> PiE_mem
2943 extensional_funcset_extend_domainI ~> PiE_fun_upd
2944 extensional_funcset_restrict_domain ~> fun_upd_in_PiE
2945 extensional_funcset_extend_domain_eq ~> PiE_insert_eq
2946 card_extensional_funcset ~> card_PiE
2947 finite_extensional_funcset ~> finite_PiE
2951 * Theory Library/FinFun: theory of almost everywhere constant
2952 functions (supersedes the AFP entry "Code Generation for Functions as
2955 * Theory Library/Phantom: generic phantom type to make a type
2956 parameter appear in a constant's type. This alternative to adding
2957 TYPE('a) as another parameter avoids unnecessary closures in generated
2960 * Theory Library/RBT_Impl: efficient construction of red-black trees
2961 from sorted associative lists. Merging two trees with rbt_union may
2962 return a structurally different tree than before. Potential
2965 * Theory Library/IArray: immutable arrays with code generation.
2967 * Theory Library/Finite_Lattice: theory of finite lattices.
2969 * HOL/Multivariate_Analysis: replaced
2971 "basis :: 'a::euclidean_space => nat => real"
2972 "\<Chi>\<Chi> :: (nat => real) => 'a::euclidean_space"
2974 on euclidean spaces by using the inner product "_ \<bullet> _" with
2975 vectors from the Basis set: "\<Chi>\<Chi> i. f i" is superseded by
2976 "SUM i : Basis. f i * r i".
2978 With this change the following constants are also changed or removed:
2980 DIM('a) :: nat ~> card (Basis :: 'a set) (is an abbreviation)
2981 a $$ i ~> inner a i (where i : Basis)
2983 \<pi>, \<pi>' removed
2985 Theorems about these constants where removed.
2989 component_le_norm ~> Basis_le_norm
2990 euclidean_eq ~> euclidean_eq_iff
2991 differential_zero_maxmin_component ~> differential_zero_maxmin_cart
2992 euclidean_simps ~> inner_simps
2993 independent_basis ~> independent_Basis
2994 span_basis ~> span_Basis
2995 in_span_basis ~> in_span_Basis
2996 norm_bound_component_le ~> norm_boound_Basis_le
2997 norm_bound_component_lt ~> norm_boound_Basis_lt
2998 component_le_infnorm ~> Basis_le_infnorm
3004 - Added simproc "measurable" to automatically prove measurability.
3006 - Added induction rules for sigma sets with disjoint union
3007 (sigma_sets_induct_disjoint) and for Borel-measurable functions
3008 (borel_measurable_induct).
3010 - Added the Daniell-Kolmogorov theorem (the existence the limit of a
3013 * HOL/Cardinals: Theories of ordinals and cardinals (supersedes the
3014 AFP entry "Ordinals_and_Cardinals").
3016 * HOL/BNF: New (co)datatype package based on bounded natural functors
3017 with support for mixed, nested recursion and interesting non-free
3020 * HOL/Finite_Set and Relation: added new set and relation operations
3021 expressed by Finite_Set.fold.
3023 * New theory HOL/Library/RBT_Set: implementation of sets by red-black
3024 trees for the code generator.
3026 * HOL/Library/RBT and HOL/Library/Mapping have been converted to
3028 possible INCOMPATIBILITY.
3030 * HOL/Set: renamed Set.project -> Set.filter
3034 *** Document preparation ***
3036 * Dropped legacy antiquotations "term_style" and "thm_style", since
3037 styles may be given as arguments to "term" and "thm" already.
3038 Discontinued legacy styles "prem1" .. "prem19".
3040 * Default LaTeX rendering for \<euro> is now based on eurosym package,
3041 instead of slightly exotic babel/greek.
3043 * Document variant NAME may use different LaTeX entry point
3044 document/root_NAME.tex if that file exists, instead of the common
3047 * Simplified custom document/build script, instead of old-style
3048 document/IsaMakefile. Minor INCOMPATIBILITY.
3053 * The default limit for maximum number of worker threads is now 8,
3054 instead of 4, in correspondence to capabilities of contemporary
3055 hardware and Poly/ML runtime system.
3057 * Type Seq.results and related operations support embedded error
3058 messages within lazy enumerations, and thus allow to provide
3059 informative errors in the absence of any usable results.
3061 * Renamed Position.str_of to Position.here to emphasize that this is a
3062 formal device to inline positions into message text, but not
3063 necessarily printing visible text.
3068 * Advanced support for Isabelle sessions and build management, see
3069 "system" manual for the chapter of that name, especially the "isabelle
3070 build" tool and its examples. The "isabelle mkroot" tool prepares
3071 session root directories for use with "isabelle build", similar to
3072 former "isabelle mkdir" for "isabelle usedir". Note that this affects
3073 document preparation as well. INCOMPATIBILITY, isabelle usedir /
3074 mkdir / make are rendered obsolete.
3076 * Discontinued obsolete Isabelle/build script, it is superseded by the
3077 regular isabelle build tool. For example:
3079 isabelle build -s -b HOL
3081 * Discontinued obsolete "isabelle makeall".
3083 * Discontinued obsolete IsaMakefile and ROOT.ML files from the
3084 Isabelle distribution, except for rudimentary src/HOL/IsaMakefile that
3085 provides some traditional targets that invoke "isabelle build". Note
3086 that this is inefficient! Applications of Isabelle/HOL involving
3087 "isabelle make" should be upgraded to use "isabelle build" directly.
3089 * The "isabelle options" tool prints Isabelle system options, as
3090 required for "isabelle build", for example.
3092 * The "isabelle logo" tool produces EPS and PDF format simultaneously.
3093 Minor INCOMPATIBILITY in command-line options.
3095 * The "isabelle install" tool has now a simpler command-line. Minor
3098 * The "isabelle components" tool helps to resolve add-on components
3099 that are not bundled, or referenced from a bare-bones repository
3100 version of Isabelle.
3102 * Settings variable ISABELLE_PLATFORM_FAMILY refers to the general
3103 platform family: "linux", "macos", "windows".
3105 * The ML system is configured as regular component, and no longer
3106 picked up from some surrounding directory. Potential INCOMPATIBILITY
3107 for home-made settings.
3109 * Improved ML runtime statistics (heap, threads, future tasks etc.).
3111 * Discontinued support for Poly/ML 5.2.1, which was the last version
3112 without exception positions and advanced ML compiler/toplevel
3115 * Discontinued special treatment of Proof General -- no longer guess
3116 PROOFGENERAL_HOME based on accidental file-system layout. Minor
3117 INCOMPATIBILITY: provide PROOFGENERAL_HOME and PROOFGENERAL_OPTIONS
3118 settings manually, or use a Proof General version that has been
3119 bundled as Isabelle component.
3123 New in Isabelle2012 (May 2012)
3124 ------------------------------
3128 * Prover IDE (PIDE) improvements:
3130 - more robust Sledgehammer integration (as before the sledgehammer
3131 command-line needs to be typed into the source buffer)
3132 - markup for bound variables
3133 - markup for types of term variables (displayed as tooltips)
3134 - support for user-defined Isar commands within the running session
3135 - improved support for Unicode outside original 16bit range
3136 e.g. glyph for \<A> (thanks to jEdit 4.5.1)
3138 * Forward declaration of outer syntax keywords within the theory
3139 header -- minor INCOMPATIBILITY for user-defined commands. Allow new
3140 commands to be used in the same theory where defined.
3142 * Auxiliary contexts indicate block structure for specifications with
3143 additional parameters and assumptions. Such unnamed contexts may be
3144 nested within other targets, like 'theory', 'locale', 'class',
3145 'instantiation' etc. Results from the local context are generalized
3146 accordingly and applied to the enclosing target context. Example:
3150 assumes xy: "x = y" and yz: "y = z"
3153 lemma my_trans: "x = z" using xy yz by simp
3159 The most basic application is to factor-out context elements of
3160 several fixes/assumes/shows theorem statements, e.g. see
3161 ~~/src/HOL/Isar_Examples/Group_Context.thy
3163 Any other local theory specification element works within the "context
3164 ... begin ... end" block as well.
3166 * Bundled declarations associate attributed fact expressions with a
3167 given name in the context. These may be later included in other
3168 contexts. This allows to manage context extensions casually, without
3169 the logical dependencies of locales and locale interpretation. See
3170 commands 'bundle', 'include', 'including' etc. in the isar-ref manual.
3172 * Commands 'lemmas' and 'theorems' allow local variables using 'for'
3173 declaration, and results are standardized before being stored. Thus
3174 old-style "standard" after instantiation or composition of facts
3175 becomes obsolete. Minor INCOMPATIBILITY, due to potential change of
3176 indices of schematic variables.
3178 * Rule attributes in local theory declarations (e.g. locale or class)
3179 are now statically evaluated: the resulting theorem is stored instead
3180 of the original expression. INCOMPATIBILITY in rare situations, where
3181 the historic accident of dynamic re-evaluation in interpretations
3184 * New tutorial "Programming and Proving in Isabelle/HOL"
3185 ("prog-prove"). It completely supersedes "A Tutorial Introduction to
3186 Structured Isar Proofs" ("isar-overview"), which has been removed. It
3187 also supersedes "Isabelle/HOL, A Proof Assistant for Higher-Order
3188 Logic" as the recommended beginners tutorial, but does not cover all
3189 of the material of that old tutorial.
3191 * Updated and extended reference manuals: "isar-ref",
3192 "implementation", "system"; reduced remaining material in old "ref"
3198 * Command 'definition' no longer exports the foundational "raw_def"
3199 into the user context. Minor INCOMPATIBILITY, may use the regular
3200 "def" result with attribute "abs_def" to imitate the old version.
3202 * Attribute "abs_def" turns an equation of the form "f x y == t" into
3203 "f == %x y. t", which ensures that "simp" or "unfold" steps always
3204 expand it. This also works for object-logic equality. (Formerly
3205 undocumented feature.)
3207 * Sort constraints are now propagated in simultaneous statements, just
3208 like type constraints. INCOMPATIBILITY in rare situations, where
3209 distinct sorts used to be assigned accidentally. For example:
3211 lemma "P (x::'a::foo)" and "Q (y::'a::bar)" -- "now illegal"
3213 lemma "P (x::'a)" and "Q (y::'a::bar)"
3214 -- "now uniform 'a::bar instead of default sort for first occurrence (!)"
3216 * Rule composition via attribute "OF" (or ML functions OF/MRS) is more
3217 tolerant against multiple unifiers, as long as the final result is
3218 unique. (As before, rules are composed in canonical right-to-left
3219 order to accommodate newly introduced premises.)
3221 * Renamed some inner syntax categories:
3227 Minor INCOMPATIBILITY. Note that in practice "num_const" or
3228 "num_position" etc. are mainly used instead (which also include
3229 position information via constraints).
3231 * Simplified configuration options for syntax ambiguity: see
3232 "syntax_ambiguity_warning" and "syntax_ambiguity_limit" in isar-ref
3233 manual. Minor INCOMPATIBILITY.
3235 * Discontinued configuration option "syntax_positions": atomic terms
3236 in parse trees are always annotated by position constraints.
3238 * Old code generator for SML and its commands 'code_module',
3239 'code_library', 'consts_code', 'types_code' have been discontinued.
3240 Use commands of the generic code generator instead. INCOMPATIBILITY.
3242 * Redundant attribute "code_inline" has been discontinued. Use
3243 "code_unfold" instead. INCOMPATIBILITY.
3245 * Dropped attribute "code_unfold_post" in favor of the its dual
3246 "code_abbrev", which yields a common pattern in definitions like
3248 definition [code_abbrev]: "f = t"
3252 * Obsolete 'types' command has been discontinued. Use 'type_synonym'
3253 instead. INCOMPATIBILITY.
3255 * Discontinued old "prems" fact, which used to refer to the accidental
3256 collection of foundational premises in the context (already marked as
3257 legacy since Isabelle2011).
3262 * Type 'a set is now a proper type constructor (just as before
3263 Isabelle2008). Definitions mem_def and Collect_def have disappeared.
3264 Non-trivial INCOMPATIBILITY. For developments keeping predicates and
3265 sets separate, it is often sufficient to rephrase some set S that has
3266 been accidentally used as predicates by "%x. x : S", and some
3267 predicate P that has been accidentally used as set by "{x. P x}".
3268 Corresponding proofs in a first step should be pruned from any
3269 tinkering with former theorems mem_def and Collect_def as far as
3272 For developments which deliberately mix predicates and sets, a
3273 planning step is necessary to determine what should become a predicate
3274 and what a set. It can be helpful to carry out that step in
3275 Isabelle2011-1 before jumping right into the current release.
3277 * Code generation by default implements sets as container type rather
3278 than predicates. INCOMPATIBILITY.
3280 * New type synonym 'a rel = ('a * 'a) set
3282 * The representation of numerals has changed. Datatype "num"
3283 represents strictly positive binary numerals, along with functions
3284 "numeral :: num => 'a" and "neg_numeral :: num => 'a" to represent
3285 positive and negated numeric literals, respectively. See also
3286 definitions in ~~/src/HOL/Num.thy. Potential INCOMPATIBILITY, some
3287 user theories may require adaptations as follows:
3289 - Theorems with number_ring or number_semiring constraints: These
3290 classes are gone; use comm_ring_1 or comm_semiring_1 instead.
3292 - Theories defining numeric types: Remove number, number_semiring,
3293 and number_ring instances. Defer all theorems about numerals until
3294 after classes one and semigroup_add have been instantiated.
3296 - Numeral-only simp rules: Replace each rule having a "number_of v"
3297 pattern with two copies, one for numeral and one for neg_numeral.
3299 - Theorems about subclasses of semiring_1 or ring_1: These classes
3300 automatically support numerals now, so more simp rules and
3301 simprocs may now apply within the proof.
3303 - Definitions and theorems using old constructors Pls/Min/Bit0/Bit1:
3304 Redefine using other integer operations.
3306 * Transfer: New package intended to generalize the existing
3307 "descending" method and related theorem attributes from the Quotient
3308 package. (Not all functionality is implemented yet, but future
3309 development will focus on Transfer as an eventual replacement for the
3310 corresponding parts of the Quotient package.)
3312 - transfer_rule attribute: Maintains a collection of transfer rules,
3313 which relate constants at two different types. Transfer rules may
3314 relate different type instances of the same polymorphic constant,
3315 or they may relate an operation on a raw type to a corresponding
3316 operation on an abstract type (quotient or subtype). For example:
3318 ((A ===> B) ===> list_all2 A ===> list_all2 B) map map
3319 (cr_int ===> cr_int ===> cr_int) (%(x,y) (u,v). (x+u, y+v)) plus_int
3321 - transfer method: Replaces a subgoal on abstract types with an
3322 equivalent subgoal on the corresponding raw types. Constants are
3323 replaced with corresponding ones according to the transfer rules.
3324 Goals are generalized over all free variables by default; this is
3325 necessary for variables whose types change, but can be overridden
3326 for specific variables with e.g. "transfer fixing: x y z". The
3327 variant transfer' method allows replacing a subgoal with one that
3328 is logically stronger (rather than equivalent).
3330 - relator_eq attribute: Collects identity laws for relators of
3331 various type constructors, e.g. "list_all2 (op =) = (op =)". The
3332 transfer method uses these lemmas to infer transfer rules for
3333 non-polymorphic constants on the fly.
3335 - transfer_prover method: Assists with proving a transfer rule for a
3336 new constant, provided the constant is defined in terms of other
3337 constants that already have transfer rules. It should be applied
3338 after unfolding the constant definitions.
3340 - HOL/ex/Transfer_Int_Nat.thy: Example theory demonstrating transfer
3341 from type nat to type int.
3343 * Lifting: New package intended to generalize the quotient_definition
3344 facility of the Quotient package; designed to work with Transfer.
3346 - lift_definition command: Defines operations on an abstract type in
3347 terms of a corresponding operation on a representation
3348 type. Example syntax:
3350 lift_definition dlist_insert :: "'a => 'a dlist => 'a dlist"
3353 Users must discharge a respectfulness proof obligation when each
3354 constant is defined. (For a type copy, i.e. a typedef with UNIV,
3355 the proof is discharged automatically.) The obligation is
3356 presented in a user-friendly, readable form; a respectfulness
3357 theorem in the standard format and a transfer rule are generated
3360 - Integration with code_abstype: For typedefs (e.g. subtypes
3361 corresponding to a datatype invariant, such as dlist),
3362 lift_definition generates a code certificate theorem and sets up
3363 code generation for each constant.
3365 - setup_lifting command: Sets up the Lifting package to work with a
3366 user-defined type. The user must provide either a quotient theorem
3367 or a type_definition theorem. The package configures transfer
3368 rules for equality and quantifiers on the type, and sets up the
3369 lift_definition command to work with the type.
3371 - Usage examples: See Quotient_Examples/Lift_DList.thy,
3372 Quotient_Examples/Lift_RBT.thy, Quotient_Examples/Lift_FSet.thy,
3373 Word/Word.thy and Library/Float.thy.
3377 - The 'quotient_type' command now supports a 'morphisms' option with
3378 rep and abs functions, similar to typedef.
3380 - 'quotient_type' sets up new types to work with the Lifting and
3381 Transfer packages, as with 'setup_lifting'.
3383 - The 'quotient_definition' command now requires the user to prove a
3384 respectfulness property at the point where the constant is
3385 defined, similar to lift_definition; INCOMPATIBILITY.
3387 - Renamed predicate 'Quotient' to 'Quotient3', and renamed theorems
3388 accordingly, INCOMPATIBILITY.
3390 * New diagnostic command 'find_unused_assms' to find potentially
3391 superfluous assumptions in theorems using Quickcheck.
3395 - Quickcheck returns variable assignments as counterexamples, which
3396 allows to reveal the underspecification of functions under test.
3397 For example, refuting "hd xs = x", it presents the variable
3398 assignment xs = [] and x = a1 as a counterexample, assuming that
3399 any property is false whenever "hd []" occurs in it.
3401 These counterexample are marked as potentially spurious, as
3402 Quickcheck also returns "xs = []" as a counterexample to the
3403 obvious theorem "hd xs = hd xs".
3405 After finding a potentially spurious counterexample, Quickcheck
3406 continues searching for genuine ones.
3408 By default, Quickcheck shows potentially spurious and genuine
3409 counterexamples. The option "genuine_only" sets quickcheck to only
3410 show genuine counterexamples.
3412 - The command 'quickcheck_generator' creates random and exhaustive
3413 value generators for a given type and operations.
3415 It generates values by using the operations as if they were
3416 constructors of that type.
3418 - Support for multisets.
3420 - Added "use_subtype" options.
3422 - Added "quickcheck_locale" configuration to specify how to process
3423 conjectures in a locale context.
3425 * Nitpick: Fixed infinite loop caused by the 'peephole_optim' option
3426 and affecting 'rat' and 'real'.
3429 - Integrated more tightly with SPASS, as described in the ITP 2012
3430 paper "More SPASS with Isabelle".
3431 - Made it try "smt" as a fallback if "metis" fails or times out.
3432 - Added support for the following provers: Alt-Ergo (via Why3 and
3433 TFF1), iProver, iProver-Eq.
3434 - Sped up the minimizer.
3435 - Added "lam_trans", "uncurry_aliases", and "minimize" options.
3436 - Renamed "slicing" ("no_slicing") option to "slice" ("dont_slice").
3437 - Renamed "sound" option to "strict".
3439 * Metis: Added possibility to specify lambda translations scheme as a
3440 parenthesized argument (e.g., "by (metis (lifting) ...)").
3442 * SMT: Renamed "smt_fixed" option to "smt_read_only_certificates".
3444 * Command 'try0': Renamed from 'try_methods'. INCOMPATIBILITY.
3446 * New "case_product" attribute to generate a case rule doing multiple
3447 case distinctions at the same time. E.g.
3449 list.exhaust [case_product nat.exhaust]
3451 produces a rule which can be used to perform case distinction on both
3454 * New "eventually_elim" method as a generalized variant of the
3455 eventually_elim* rules. Supports structured proofs.
3457 * Typedef with implicit set definition is considered legacy. Use
3458 "typedef (open)" form instead, which will eventually become the
3461 * Record: code generation can be switched off manually with
3463 declare [[record_coden = false]] -- "default true"
3465 * Datatype: type parameters allow explicit sort constraints.
3467 * Concrete syntax for case expressions includes constraints for source
3468 positions, and thus produces Prover IDE markup for its bindings.
3469 INCOMPATIBILITY for old-style syntax translations that augment the
3470 pattern notation; e.g. see src/HOL/HOLCF/One.thy for translations of
3473 * Clarified attribute "mono_set": pure declaration without modifying
3474 the result of the fact expression.
3476 * More default pred/set conversions on a couple of relation operations
3477 and predicates. Added powers of predicate relations. Consolidation
3478 of some relation theorems:
3480 converse_def ~> converse_unfold
3481 rel_comp_def ~> relcomp_unfold
3482 symp_def ~> (modified, use symp_def and sym_def instead)
3483 transp_def ~> transp_trans
3484 Domain_def ~> Domain_unfold
3485 Range_def ~> Domain_converse [symmetric]
3487 Generalized theorems INF_INT_eq, INF_INT_eq2, SUP_UN_eq, SUP_UN_eq2.
3489 See theory "Relation" for examples for making use of pred/set
3490 conversions by means of attributes "to_set" and "to_pred".
3494 * Renamed facts about the power operation on relations, i.e., relpow
3495 to match the constant's name:
3497 rel_pow_1 ~> relpow_1
3498 rel_pow_0_I ~> relpow_0_I
3499 rel_pow_Suc_I ~> relpow_Suc_I
3500 rel_pow_Suc_I2 ~> relpow_Suc_I2
3501 rel_pow_0_E ~> relpow_0_E
3502 rel_pow_Suc_E ~> relpow_Suc_E
3503 rel_pow_E ~> relpow_E
3504 rel_pow_Suc_D2 ~> relpow_Suc_D2
3505 rel_pow_Suc_E2 ~> relpow_Suc_E2
3506 rel_pow_Suc_D2' ~> relpow_Suc_D2'
3507 rel_pow_E2 ~> relpow_E2
3508 rel_pow_add ~> relpow_add
3509 rel_pow_commute ~> relpow
3510 rel_pow_empty ~> relpow_empty:
3511 rtrancl_imp_UN_rel_pow ~> rtrancl_imp_UN_relpow
3512 rel_pow_imp_rtrancl ~> relpow_imp_rtrancl
3513 rtrancl_is_UN_rel_pow ~> rtrancl_is_UN_relpow
3514 rtrancl_imp_rel_pow ~> rtrancl_imp_relpow
3515 rel_pow_fun_conv ~> relpow_fun_conv
3516 rel_pow_finite_bounded1 ~> relpow_finite_bounded1
3517 rel_pow_finite_bounded ~> relpow_finite_bounded
3518 rtrancl_finite_eq_rel_pow ~> rtrancl_finite_eq_relpow
3519 trancl_finite_eq_rel_pow ~> trancl_finite_eq_relpow
3520 single_valued_rel_pow ~> single_valued_relpow
3524 * Theory Relation: Consolidated constant name for relation composition
3525 and corresponding theorem names:
3527 - Renamed constant rel_comp to relcomp.
3529 - Dropped abbreviation pred_comp. Use relcompp instead.
3533 rel_compI ~> relcompI
3534 rel_compEpair ~> relcompEpair
3535 rel_compE ~> relcompE
3536 pred_comp_rel_comp_eq ~> relcompp_relcomp_eq
3537 rel_comp_empty1 ~> relcomp_empty1
3538 rel_comp_mono ~> relcomp_mono
3539 rel_comp_subset_Sigma ~> relcomp_subset_Sigma
3540 rel_comp_distrib ~> relcomp_distrib
3541 rel_comp_distrib2 ~> relcomp_distrib2
3542 rel_comp_UNION_distrib ~> relcomp_UNION_distrib
3543 rel_comp_UNION_distrib2 ~> relcomp_UNION_distrib2
3544 single_valued_rel_comp ~> single_valued_relcomp
3545 rel_comp_def ~> relcomp_unfold
3546 converse_rel_comp ~> converse_relcomp
3547 pred_compI ~> relcomppI
3548 pred_compE ~> relcomppE
3549 pred_comp_bot1 ~> relcompp_bot1
3550 pred_comp_bot2 ~> relcompp_bot2
3551 transp_pred_comp_less_eq ~> transp_relcompp_less_eq
3552 pred_comp_mono ~> relcompp_mono
3553 pred_comp_distrib ~> relcompp_distrib
3554 pred_comp_distrib2 ~> relcompp_distrib2
3555 converse_pred_comp ~> converse_relcompp
3557 finite_rel_comp ~> finite_relcomp
3559 set_rel_comp ~> set_relcomp
3563 * Theory Divides: Discontinued redundant theorems about div and mod.
3564 INCOMPATIBILITY, use the corresponding generic theorems instead.
3566 DIVISION_BY_ZERO ~> div_by_0, mod_by_0
3567 zdiv_self ~> div_self
3568 zmod_self ~> mod_self
3571 zdiv_zmod_equality ~> div_mod_equality2
3572 zdiv_zmod_equality2 ~> div_mod_equality
3573 zmod_zdiv_trivial ~> mod_div_trivial
3574 zdiv_zminus_zminus ~> div_minus_minus
3575 zmod_zminus_zminus ~> mod_minus_minus
3576 zdiv_zminus2 ~> div_minus_right
3577 zmod_zminus2 ~> mod_minus_right
3578 zdiv_minus1_right ~> div_minus1_right
3579 zmod_minus1_right ~> mod_minus1_right
3580 zdvd_mult_div_cancel ~> dvd_mult_div_cancel
3581 zmod_zmult1_eq ~> mod_mult_right_eq
3582 zpower_zmod ~> power_mod
3583 zdvd_zmod ~> dvd_mod
3584 zdvd_zmod_imp_zdvd ~> dvd_mod_imp_dvd
3585 mod_mult_distrib ~> mult_mod_left
3586 mod_mult_distrib2 ~> mult_mod_right
3588 * Removed redundant theorems nat_mult_2 and nat_mult_2_right; use
3589 generic mult_2 and mult_2_right instead. INCOMPATIBILITY.
3591 * Finite_Set.fold now qualified. INCOMPATIBILITY.
3593 * Consolidated theorem names concerning fold combinators:
3595 inf_INFI_fold_inf ~> inf_INF_fold_inf
3596 sup_SUPR_fold_sup ~> sup_SUP_fold_sup
3597 INFI_fold_inf ~> INF_fold_inf
3598 SUPR_fold_sup ~> SUP_fold_sup
3599 union_set ~> union_set_fold
3600 minus_set ~> minus_set_fold
3601 INFI_set_fold ~> INF_set_fold
3602 SUPR_set_fold ~> SUP_set_fold
3603 INF_code ~> INF_set_foldr
3604 SUP_code ~> SUP_set_foldr
3605 foldr.simps ~> foldr.simps (in point-free formulation)
3606 foldr_fold_rev ~> foldr_conv_fold
3607 foldl_fold ~> foldl_conv_fold
3608 foldr_foldr ~> foldr_conv_foldl
3609 foldl_foldr ~> foldl_conv_foldr
3610 fold_set_remdups ~> fold_set_fold_remdups
3611 fold_set ~> fold_set_fold
3612 fold1_set ~> fold1_set_fold
3616 * Dropped rarely useful theorems concerning fold combinators:
3617 foldl_apply, foldl_fun_comm, foldl_rev, fold_weak_invariant,
3618 rev_foldl_cons, fold_set_remdups, fold_set, fold_set1,
3619 concat_conv_foldl, foldl_weak_invariant, foldl_invariant,
3620 foldr_invariant, foldl_absorb0, foldl_foldr1_lemma, foldl_foldr1,
3621 listsum_conv_fold, listsum_foldl, sort_foldl_insort, foldl_assoc,
3622 foldr_conv_foldl, start_le_sum, elem_le_sum, sum_eq_0_conv.
3623 INCOMPATIBILITY. For the common phrases "%xs. List.foldr plus xs 0"
3624 and "List.foldl plus 0", prefer "List.listsum". Otherwise it can be
3625 useful to boil down "List.foldr" and "List.foldl" to "List.fold" by
3626 unfolding "foldr_conv_fold" and "foldl_conv_fold".
3628 * Dropped lemmas minus_set_foldr, union_set_foldr, union_coset_foldr,
3629 inter_coset_foldr, Inf_fin_set_foldr, Sup_fin_set_foldr,
3630 Min_fin_set_foldr, Max_fin_set_foldr, Inf_set_foldr, Sup_set_foldr,
3631 INF_set_foldr, SUP_set_foldr. INCOMPATIBILITY. Prefer corresponding
3632 lemmas over fold rather than foldr, or make use of lemmas
3633 fold_conv_foldr and fold_rev.
3635 * Congruence rules Option.map_cong and Option.bind_cong for recursion
3636 through option types.
3638 * "Transitive_Closure.ntrancl": bounded transitive closure on
3641 * Constant "Set.not_member" now qualified. INCOMPATIBILITY.
3643 * Theory Int: Discontinued many legacy theorems specific to type int.
3644 INCOMPATIBILITY, use the corresponding generic theorems instead.
3646 zminus_zminus ~> minus_minus
3647 zminus_0 ~> minus_zero
3648 zminus_zadd_distrib ~> minus_add_distrib
3649 zadd_commute ~> add_commute
3650 zadd_assoc ~> add_assoc
3651 zadd_left_commute ~> add_left_commute
3654 zadd_0 ~> add_0_left
3655 zadd_0_right ~> add_0_right
3656 zadd_zminus_inverse2 ~> left_minus
3657 zmult_zminus ~> mult_minus_left
3658 zmult_commute ~> mult_commute
3659 zmult_assoc ~> mult_assoc
3660 zadd_zmult_distrib ~> left_distrib
3661 zadd_zmult_distrib2 ~> right_distrib
3662 zdiff_zmult_distrib ~> left_diff_distrib
3663 zdiff_zmult_distrib2 ~> right_diff_distrib
3664 zmult_1 ~> mult_1_left
3665 zmult_1_right ~> mult_1_right
3666 zle_refl ~> order_refl
3667 zle_trans ~> order_trans
3668 zle_antisym ~> order_antisym
3669 zle_linear ~> linorder_linear
3670 zless_linear ~> linorder_less_linear
3671 zadd_left_mono ~> add_left_mono
3672 zadd_strict_right_mono ~> add_strict_right_mono
3673 zadd_zless_mono ~> add_less_le_mono
3674 int_0_less_1 ~> zero_less_one
3675 int_0_neq_1 ~> zero_neq_one
3677 zpower_zadd_distrib ~> power_add
3678 zero_less_zpower_abs_iff ~> zero_less_power_abs_iff
3679 zero_le_zpower_abs ~> zero_le_power_abs
3681 * Theory Deriv: Renamed
3683 DERIV_nonneg_imp_nonincreasing ~> DERIV_nonneg_imp_nondecreasing
3685 * Theory Library/Multiset: Improved code generation of multisets.
3687 * Theory HOL/Library/Set_Algebras: Addition and multiplication on sets
3688 are expressed via type classes again. The special syntax
3689 \<oplus>/\<otimes> has been replaced by plain +/*. Removed constant
3690 setsum_set, which is now subsumed by Big_Operators.setsum.
3693 * Theory HOL/Library/Diagonalize has been removed. INCOMPATIBILITY,
3694 use theory HOL/Library/Nat_Bijection instead.
3696 * Theory HOL/Library/RBT_Impl: Backing implementation of red-black
3697 trees is now inside a type class context. Names of affected
3698 operations and lemmas have been prefixed by rbt_. INCOMPATIBILITY for
3699 theories working directly with raw red-black trees, adapt the names as
3703 bulkload -> rbt_bulkload
3704 del_from_left -> rbt_del_from_left
3705 del_from_right -> rbt_del_from_right
3707 delete -> rbt_delete
3709 insert -> rbt_insert
3710 insertw -> rbt_insert_with
3711 insert_with_key -> rbt_insert_with_key
3712 map_entry -> rbt_map_entry
3713 lookup -> rbt_lookup
3714 sorted -> rbt_sorted
3715 tree_greater -> rbt_greater
3716 tree_less -> rbt_less
3717 tree_less_symbol -> rbt_less_symbol
3719 union_with -> rbt_union_with
3720 union_with_key -> rbt_union_with_key
3723 balance_left_sorted -> balance_left_rbt_sorted
3724 balance_left_tree_greater -> balance_left_rbt_greater
3725 balance_left_tree_less -> balance_left_rbt_less
3726 balance_right_sorted -> balance_right_rbt_sorted
3727 balance_right_tree_greater -> balance_right_rbt_greater
3728 balance_right_tree_less -> balance_right_rbt_less
3729 balance_sorted -> balance_rbt_sorted
3730 balance_tree_greater -> balance_rbt_greater
3731 balance_tree_less -> balance_rbt_less
3732 bulkload_is_rbt -> rbt_bulkload_is_rbt
3733 combine_sorted -> combine_rbt_sorted
3734 combine_tree_greater -> combine_rbt_greater
3735 combine_tree_less -> combine_rbt_less
3736 delete_in_tree -> rbt_delete_in_tree
3737 delete_is_rbt -> rbt_delete_is_rbt
3738 del_from_left_tree_greater -> rbt_del_from_left_rbt_greater
3739 del_from_left_tree_less -> rbt_del_from_left_rbt_less
3740 del_from_right_tree_greater -> rbt_del_from_right_rbt_greater
3741 del_from_right_tree_less -> rbt_del_from_right_rbt_less
3742 del_in_tree -> rbt_del_in_tree
3743 del_inv1_inv2 -> rbt_del_inv1_inv2
3744 del_sorted -> rbt_del_rbt_sorted
3745 del_tree_greater -> rbt_del_rbt_greater
3746 del_tree_less -> rbt_del_rbt_less
3747 dom_lookup_Branch -> dom_rbt_lookup_Branch
3748 entries_lookup -> entries_rbt_lookup
3749 finite_dom_lookup -> finite_dom_rbt_lookup
3750 insert_sorted -> rbt_insert_rbt_sorted
3751 insertw_is_rbt -> rbt_insertw_is_rbt
3752 insertwk_is_rbt -> rbt_insertwk_is_rbt
3753 insertwk_sorted -> rbt_insertwk_rbt_sorted
3754 insertw_sorted -> rbt_insertw_rbt_sorted
3755 ins_sorted -> ins_rbt_sorted
3756 ins_tree_greater -> ins_rbt_greater
3757 ins_tree_less -> ins_rbt_less
3758 is_rbt_sorted -> is_rbt_rbt_sorted
3759 lookup_balance -> rbt_lookup_balance
3760 lookup_bulkload -> rbt_lookup_rbt_bulkload
3761 lookup_delete -> rbt_lookup_rbt_delete
3762 lookup_Empty -> rbt_lookup_Empty
3763 lookup_from_in_tree -> rbt_lookup_from_in_tree
3764 lookup_in_tree -> rbt_lookup_in_tree
3765 lookup_ins -> rbt_lookup_ins
3766 lookup_insert -> rbt_lookup_rbt_insert
3767 lookup_insertw -> rbt_lookup_rbt_insertw
3768 lookup_insertwk -> rbt_lookup_rbt_insertwk
3769 lookup_keys -> rbt_lookup_keys
3770 lookup_map -> rbt_lookup_map
3771 lookup_map_entry -> rbt_lookup_rbt_map_entry
3772 lookup_tree_greater -> rbt_lookup_rbt_greater
3773 lookup_tree_less -> rbt_lookup_rbt_less
3774 lookup_union -> rbt_lookup_rbt_union
3775 map_entry_color_of -> rbt_map_entry_color_of
3776 map_entry_inv1 -> rbt_map_entry_inv1
3777 map_entry_inv2 -> rbt_map_entry_inv2
3778 map_entry_is_rbt -> rbt_map_entry_is_rbt
3779 map_entry_sorted -> rbt_map_entry_rbt_sorted
3780 map_entry_tree_greater -> rbt_map_entry_rbt_greater
3781 map_entry_tree_less -> rbt_map_entry_rbt_less
3782 map_tree_greater -> map_rbt_greater
3783 map_tree_less -> map_rbt_less
3784 map_sorted -> map_rbt_sorted
3785 paint_sorted -> paint_rbt_sorted
3786 paint_lookup -> paint_rbt_lookup
3787 paint_tree_greater -> paint_rbt_greater
3788 paint_tree_less -> paint_rbt_less
3789 sorted_entries -> rbt_sorted_entries
3790 tree_greater_eq_trans -> rbt_greater_eq_trans
3791 tree_greater_nit -> rbt_greater_nit
3792 tree_greater_prop -> rbt_greater_prop
3793 tree_greater_simps -> rbt_greater_simps
3794 tree_greater_trans -> rbt_greater_trans
3795 tree_less_eq_trans -> rbt_less_eq_trans
3796 tree_less_nit -> rbt_less_nit
3797 tree_less_prop -> rbt_less_prop
3798 tree_less_simps -> rbt_less_simps
3799 tree_less_trans -> rbt_less_trans
3800 tree_ord_props -> rbt_ord_props
3801 union_Branch -> rbt_union_Branch
3802 union_is_rbt -> rbt_union_is_rbt
3803 unionw_is_rbt -> rbt_unionw_is_rbt
3804 unionwk_is_rbt -> rbt_unionwk_is_rbt
3805 unionwk_sorted -> rbt_unionwk_rbt_sorted
3807 * Theory HOL/Library/Float: Floating point numbers are now defined as
3808 a subset of the real numbers. All operations are defined using the
3809 lifing-framework and proofs use the transfer method. INCOMPATIBILITY.
3816 round_down -> float_round_down
3817 round_up -> float_round_up
3821 ceiling_fl, lb_mult, lb_mod, ub_mult, ub_mod
3824 abs_float_def -> Float.compute_float_abs
3825 bitlen_ge0 -> bitlen_nonneg
3826 bitlen.simps -> Float.compute_bitlen
3827 float_components -> Float_mantissa_exponent
3828 float_divl.simps -> Float.compute_float_divl
3829 float_divr.simps -> Float.compute_float_divr
3830 float_eq_odd -> mult_powr_eq_mult_powr_iff
3831 float_power -> real_of_float_power
3832 lapprox_posrat_def -> Float.compute_lapprox_posrat
3833 lapprox_rat.simps -> Float.compute_lapprox_rat
3834 le_float_def' -> Float.compute_float_le
3835 le_float_def -> less_eq_float.rep_eq
3836 less_float_def' -> Float.compute_float_less
3837 less_float_def -> less_float.rep_eq
3838 normfloat_def -> Float.compute_normfloat
3839 normfloat_imp_odd_or_zero -> mantissa_not_dvd and mantissa_noteq_0
3840 normfloat -> normfloat_def
3841 normfloat_unique -> use normfloat_def
3842 number_of_float_Float -> Float.compute_float_numeral, Float.compute_float_neg_numeral
3843 one_float_def -> Float.compute_float_one
3844 plus_float_def -> Float.compute_float_plus
3845 rapprox_posrat_def -> Float.compute_rapprox_posrat
3846 rapprox_rat.simps -> Float.compute_rapprox_rat
3847 real_of_float_0 -> zero_float.rep_eq
3848 real_of_float_1 -> one_float.rep_eq
3849 real_of_float_abs -> abs_float.rep_eq
3850 real_of_float_add -> plus_float.rep_eq
3851 real_of_float_minus -> uminus_float.rep_eq
3852 real_of_float_mult -> times_float.rep_eq
3853 real_of_float_simp -> Float.rep_eq
3854 real_of_float_sub -> minus_float.rep_eq
3855 round_down.simps -> Float.compute_float_round_down
3856 round_up.simps -> Float.compute_float_round_up
3857 times_float_def -> Float.compute_float_times
3858 uminus_float_def -> Float.compute_float_uminus
3859 zero_float_def -> Float.compute_float_zero
3861 Lemmas not necessary anymore, use the transfer method:
3862 bitlen_B0, bitlen_B1, bitlen_ge1, bitlen_Min, bitlen_Pls, float_divl,
3863 float_divr, float_le_simp, float_less1_mantissa_bound,
3864 float_less_simp, float_less_zero, float_le_zero,
3865 float_pos_less1_e_neg, float_pos_m_pos, float_split, float_split2,
3866 floor_pos_exp, lapprox_posrat, lapprox_posrat_bottom, lapprox_rat,
3867 lapprox_rat_bottom, normalized_float, rapprox_posrat,
3868 rapprox_posrat_le1, rapprox_rat, real_of_float_ge0_exp,
3869 real_of_float_neg_exp, real_of_float_nge0_exp, round_down floor_fl,
3870 round_up, zero_le_float, zero_less_float
3872 * New theory HOL/Library/DAList provides an abstract type for
3873 association lists with distinct keys.
3875 * Session HOL/IMP: Added new theory of abstract interpretation of
3878 * Session HOL-Import: Re-implementation from scratch is faster,
3879 simpler, and more scalable. Requires a proof bundle, which is
3880 available as an external component. Discontinued old (and mostly
3881 dead) Importer for HOL4 and HOL Light. INCOMPATIBILITY.
3883 * Session HOL-Word: Discontinued many redundant theorems specific to
3884 type 'a word. INCOMPATIBILITY, use the corresponding generic theorems
3887 word_sub_alt ~> word_sub_wi
3888 word_add_alt ~> word_add_def
3889 word_mult_alt ~> word_mult_def
3890 word_minus_alt ~> word_minus_def
3891 word_0_alt ~> word_0_wi
3892 word_1_alt ~> word_1_wi
3893 word_add_0 ~> add_0_left
3894 word_add_0_right ~> add_0_right
3895 word_mult_1 ~> mult_1_left
3896 word_mult_1_right ~> mult_1_right
3897 word_add_commute ~> add_commute
3898 word_add_assoc ~> add_assoc
3899 word_add_left_commute ~> add_left_commute
3900 word_mult_commute ~> mult_commute
3901 word_mult_assoc ~> mult_assoc
3902 word_mult_left_commute ~> mult_left_commute
3903 word_left_distrib ~> left_distrib
3904 word_right_distrib ~> right_distrib
3905 word_left_minus ~> left_minus
3906 word_diff_0_right ~> diff_0_right
3907 word_diff_self ~> diff_self
3908 word_sub_def ~> diff_minus
3909 word_diff_minus ~> diff_minus
3910 word_add_ac ~> add_ac
3911 word_mult_ac ~> mult_ac
3912 word_plus_ac0 ~> add_0_left add_0_right add_ac
3913 word_times_ac1 ~> mult_1_left mult_1_right mult_ac
3914 word_order_trans ~> order_trans
3915 word_order_refl ~> order_refl
3916 word_order_antisym ~> order_antisym
3917 word_order_linear ~> linorder_linear
3918 lenw1_zero_neq_one ~> zero_neq_one
3919 word_number_of_eq ~> number_of_eq
3920 word_of_int_add_hom ~> wi_hom_add
3921 word_of_int_sub_hom ~> wi_hom_sub
3922 word_of_int_mult_hom ~> wi_hom_mult
3923 word_of_int_minus_hom ~> wi_hom_neg
3924 word_of_int_succ_hom ~> wi_hom_succ
3925 word_of_int_pred_hom ~> wi_hom_pred
3926 word_of_int_0_hom ~> word_0_wi
3927 word_of_int_1_hom ~> word_1_wi
3929 * Session HOL-Word: New proof method "word_bitwise" for splitting
3930 machine word equalities and inequalities into logical circuits,
3931 defined in HOL/Word/WordBitwise.thy. Supports addition, subtraction,
3932 multiplication, shifting by constants, bitwise operators and numeric
3933 constants. Requires fixed-length word types, not 'a word. Solves
3934 many standard word identities outright and converts more into first
3935 order problems amenable to blast or similar. See also examples in
3936 HOL/Word/Examples/WordExamples.thy.
3938 * Session HOL-Probability: Introduced the type "'a measure" to
3939 represent measures, this replaces the records 'a algebra and 'a
3940 measure_space. The locales based on subset_class now have two
3941 locale-parameters the space \<Omega> and the set of measurable sets M.
3942 The product of probability spaces uses now the same constant as the
3943 finite product of sigma-finite measure spaces "PiM :: ('i => 'a)
3944 measure". Most constants are defined now outside of locales and gain
3945 an additional parameter, like null_sets, almost_eventually or \<mu>'.
3946 Measure space constructions for distributions and densities now got
3947 their own constants distr and density. Instead of using locales to
3948 describe measure spaces with a finite space, the measure count_space
3949 and point_measure is introduced. INCOMPATIBILITY.
3953 finite_measure.\<mu>' -> measure
3954 product_algebra_generator -> prod_algebra
3955 product_prob_space.emb -> prod_emb
3956 product_prob_space.infprod_algebra -> PiM
3959 completeable_measure_space
3960 finite_measure_space
3962 finite_product_finite_prob_space
3963 finite_product_sigma_algebra
3964 finite_sigma_algebra
3966 pair_finite_prob_space
3967 pair_finite_sigma_algebra
3970 product_sigma_algebra
3974 distribution -> use distr measure, or distributed predicate
3976 joint_distribution -> use distr measure, or distributed predicate
3977 pair_measure_generator
3978 product_prob_space.infprod_algebra -> use PiM
3981 Replacement theorems:
3982 finite_additivity_sufficient -> ring_of_sets.countably_additiveI_finite
3983 finite_measure.empty_measure -> measure_empty
3984 finite_measure.finite_continuity_from_above -> finite_measure.finite_Lim_measure_decseq
3985 finite_measure.finite_continuity_from_below -> finite_measure.finite_Lim_measure_incseq
3986 finite_measure.finite_measure_countably_subadditive -> finite_measure.finite_measure_subadditive_countably
3987 finite_measure.finite_measure_eq -> finite_measure.emeasure_eq_measure
3988 finite_measure.finite_measure -> finite_measure.emeasure_finite
3989 finite_measure.finite_measure_finite_singleton -> finite_measure.finite_measure_eq_setsum_singleton
3990 finite_measure.positive_measure' -> measure_nonneg
3991 finite_measure.real_measure -> finite_measure.emeasure_real
3992 finite_product_prob_space.finite_measure_times -> finite_product_prob_space.finite_measure_PiM_emb
3993 finite_product_sigma_algebra.in_P -> sets_PiM_I_finite
3994 finite_product_sigma_algebra.P_empty -> space_PiM_empty, sets_PiM_empty
3995 information_space.conditional_entropy_eq -> information_space.conditional_entropy_simple_distributed
3996 information_space.conditional_entropy_positive -> information_space.conditional_entropy_nonneg_simple
3997 information_space.conditional_mutual_information_eq_mutual_information -> information_space.conditional_mutual_information_eq_mutual_information_simple
3998 information_space.conditional_mutual_information_generic_positive -> information_space.conditional_mutual_information_nonneg_simple
3999 information_space.conditional_mutual_information_positive -> information_space.conditional_mutual_information_nonneg_simple
4000 information_space.entropy_commute -> information_space.entropy_commute_simple
4001 information_space.entropy_eq -> information_space.entropy_simple_distributed
4002 information_space.entropy_generic_eq -> information_space.entropy_simple_distributed
4003 information_space.entropy_positive -> information_space.entropy_nonneg_simple
4004 information_space.entropy_uniform_max -> information_space.entropy_uniform
4005 information_space.KL_eq_0_imp -> information_space.KL_eq_0_iff_eq
4006 information_space.KL_eq_0 -> information_space.KL_same_eq_0
4007 information_space.KL_ge_0 -> information_space.KL_nonneg
4008 information_space.mutual_information_eq -> information_space.mutual_information_simple_distributed
4009 information_space.mutual_information_positive -> information_space.mutual_information_nonneg_simple
4010 Int_stable_cuboids -> Int_stable_atLeastAtMost
4011 Int_stable_product_algebra_generator -> positive_integral
4012 measure_preserving -> equality "distr M N f = N" "f : measurable M N"
4013 measure_space.additive -> emeasure_additive
4014 measure_space.AE_iff_null_set -> AE_iff_null
4015 measure_space.almost_everywhere_def -> eventually_ae_filter
4016 measure_space.almost_everywhere_vimage -> AE_distrD
4017 measure_space.continuity_from_above -> INF_emeasure_decseq
4018 measure_space.continuity_from_above_Lim -> Lim_emeasure_decseq
4019 measure_space.continuity_from_below_Lim -> Lim_emeasure_incseq
4020 measure_space.continuity_from_below -> SUP_emeasure_incseq
4021 measure_space_density -> emeasure_density
4022 measure_space.density_is_absolutely_continuous -> absolutely_continuousI_density
4023 measure_space.integrable_vimage -> integrable_distr
4024 measure_space.integral_translated_density -> integral_density
4025 measure_space.integral_vimage -> integral_distr
4026 measure_space.measure_additive -> plus_emeasure
4027 measure_space.measure_compl -> emeasure_compl
4028 measure_space.measure_countable_increasing -> emeasure_countable_increasing
4029 measure_space.measure_countably_subadditive -> emeasure_subadditive_countably
4030 measure_space.measure_decseq -> decseq_emeasure
4031 measure_space.measure_Diff -> emeasure_Diff
4032 measure_space.measure_Diff_null_set -> emeasure_Diff_null_set
4033 measure_space.measure_eq_0 -> emeasure_eq_0
4034 measure_space.measure_finitely_subadditive -> emeasure_subadditive_finite
4035 measure_space.measure_finite_singleton -> emeasure_eq_setsum_singleton
4036 measure_space.measure_incseq -> incseq_emeasure
4037 measure_space.measure_insert -> emeasure_insert
4038 measure_space.measure_mono -> emeasure_mono
4039 measure_space.measure_not_negative -> emeasure_not_MInf
4040 measure_space.measure_preserving_Int_stable -> measure_eqI_generator_eq
4041 measure_space.measure_setsum -> setsum_emeasure
4042 measure_space.measure_setsum_split -> setsum_emeasure_cover
4043 measure_space.measure_space_vimage -> emeasure_distr
4044 measure_space.measure_subadditive_finite -> emeasure_subadditive_finite
4045 measure_space.measure_subadditive -> subadditive
4046 measure_space.measure_top -> emeasure_space
4047 measure_space.measure_UN_eq_0 -> emeasure_UN_eq_0
4048 measure_space.measure_Un_null_set -> emeasure_Un_null_set
4049 measure_space.positive_integral_translated_density -> positive_integral_density
4050 measure_space.positive_integral_vimage -> positive_integral_distr
4051 measure_space.real_continuity_from_above -> Lim_measure_decseq
4052 measure_space.real_continuity_from_below -> Lim_measure_incseq
4053 measure_space.real_measure_countably_subadditive -> measure_subadditive_countably
4054 measure_space.real_measure_Diff -> measure_Diff
4055 measure_space.real_measure_finite_Union -> measure_finite_Union
4056 measure_space.real_measure_setsum_singleton -> measure_eq_setsum_singleton
4057 measure_space.real_measure_subadditive -> measure_subadditive
4058 measure_space.real_measure_Union -> measure_Union
4059 measure_space.real_measure_UNION -> measure_UNION
4060 measure_space.simple_function_vimage -> simple_function_comp
4061 measure_space.simple_integral_vimage -> simple_integral_distr
4062 measure_space.simple_integral_vimage -> simple_integral_distr
4063 measure_unique_Int_stable -> measure_eqI_generator_eq
4064 measure_unique_Int_stable_vimage -> measure_eqI_generator_eq
4065 pair_sigma_algebra.measurable_cut_fst -> sets_Pair1
4066 pair_sigma_algebra.measurable_cut_snd -> sets_Pair2
4067 pair_sigma_algebra.measurable_pair_image_fst -> measurable_Pair1
4068 pair_sigma_algebra.measurable_pair_image_snd -> measurable_Pair2
4069 pair_sigma_algebra.measurable_product_swap -> measurable_pair_swap_iff
4070 pair_sigma_algebra.pair_sigma_algebra_measurable -> measurable_pair_swap
4071 pair_sigma_algebra.pair_sigma_algebra_swap_measurable -> measurable_pair_swap'
4072 pair_sigma_algebra.sets_swap -> sets_pair_swap
4073 pair_sigma_finite.measure_cut_measurable_fst -> pair_sigma_finite.measurable_emeasure_Pair1
4074 pair_sigma_finite.measure_cut_measurable_snd -> pair_sigma_finite.measurable_emeasure_Pair2
4075 pair_sigma_finite.measure_preserving_swap -> pair_sigma_finite.distr_pair_swap
4076 pair_sigma_finite.pair_measure_alt2 -> pair_sigma_finite.emeasure_pair_measure_alt2
4077 pair_sigma_finite.pair_measure_alt -> pair_sigma_finite.emeasure_pair_measure_alt
4078 pair_sigma_finite.pair_measure_times -> pair_sigma_finite.emeasure_pair_measure_Times
4079 prob_space.indep_distribution_eq_measure -> prob_space.indep_vars_iff_distr_eq_PiM
4080 prob_space.indep_var_distributionD -> prob_space.indep_var_distribution_eq
4081 prob_space.measure_space_1 -> prob_space.emeasure_space_1
4082 prob_space.prob_space_vimage -> prob_space_distr
4083 prob_space.random_variable_restrict -> measurable_restrict
4084 prob_space_unique_Int_stable -> measure_eqI_prob_space
4085 product_algebraE -> prod_algebraE_all
4086 product_algebra_generator_der -> prod_algebra_eq_finite
4087 product_algebra_generator_into_space -> prod_algebra_sets_into_space
4088 product_algebraI -> sets_PiM_I_finite
4089 product_measure_exists -> product_sigma_finite.sigma_finite
4090 product_prob_space.finite_index_eq_finite_product -> product_prob_space.sets_PiM_generator
4091 product_prob_space.finite_measure_infprod_emb_Pi -> product_prob_space.measure_PiM_emb
4092 product_prob_space.infprod_spec -> product_prob_space.emeasure_PiM_emb_not_empty
4093 product_prob_space.measurable_component -> measurable_component_singleton
4094 product_prob_space.measurable_emb -> measurable_prod_emb
4095 product_prob_space.measurable_into_infprod_algebra -> measurable_PiM_single
4096 product_prob_space.measurable_singleton_infprod -> measurable_component_singleton
4097 product_prob_space.measure_emb -> emeasure_prod_emb
4098 product_prob_space.measure_preserving_restrict -> product_prob_space.distr_restrict
4099 product_sigma_algebra.product_algebra_into_space -> space_closed
4100 product_sigma_finite.measure_fold -> product_sigma_finite.distr_merge
4101 product_sigma_finite.measure_preserving_component_singelton -> product_sigma_finite.distr_singleton
4102 product_sigma_finite.measure_preserving_merge -> product_sigma_finite.distr_merge
4103 sequence_space.measure_infprod -> sequence_space.measure_PiM_countable
4104 sets_product_algebra -> sets_PiM
4105 sigma_algebra.measurable_sigma -> measurable_measure_of
4106 sigma_finite_measure.disjoint_sigma_finite -> sigma_finite_disjoint
4107 sigma_finite_measure.RN_deriv_vimage -> sigma_finite_measure.RN_deriv_distr
4108 sigma_product_algebra_sigma_eq -> sigma_prod_algebra_sigma_eq
4109 space_product_algebra -> space_PiM
4111 * Session HOL-TPTP: support to parse and import TPTP problems (all
4112 languages) into Isabelle/HOL.
4117 * New "case_product" attribute (see HOL).
4122 * Greater support for structured proofs involving induction or case
4125 * Much greater use of mathematical symbols.
4127 * Removal of many ML theorem bindings. INCOMPATIBILITY.
4132 * Antiquotation @{keyword "name"} produces a parser for outer syntax
4133 from a minor keyword introduced via theory header declaration.
4135 * Antiquotation @{command_spec "name"} produces the
4136 Outer_Syntax.command_spec from a major keyword introduced via theory
4137 header declaration; it can be passed to Outer_Syntax.command etc.
4139 * Local_Theory.define no longer hard-wires default theorem name
4140 "foo_def", but retains the binding as given. If that is Binding.empty
4141 / Attrib.empty_binding, the result is not registered as user-level
4142 fact. The Local_Theory.define_internal variant allows to specify a
4143 non-empty name (used for the foundation in the background theory),
4144 while omitting the fact binding in the user-context. Potential
4145 INCOMPATIBILITY for derived definitional packages: need to specify
4146 naming policy for primitive definitions more explicitly.
4148 * Renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in
4149 conformance with similar operations in structure Term and Logic.
4151 * Antiquotation @{attributes [...]} embeds attribute source
4152 representation into the ML text, which is particularly useful with
4153 declarations like Local_Theory.note.
4155 * Structure Proof_Context follows standard naming scheme. Old
4156 ProofContext has been discontinued. INCOMPATIBILITY.
4158 * Refined Local_Theory.declaration {syntax, pervasive}, with subtle
4159 change of semantics: update is applied to auxiliary local theory
4162 * Modernized some old-style infix operations:
4164 addeqcongs ~> Simplifier.add_eqcong
4165 deleqcongs ~> Simplifier.del_eqcong
4166 addcongs ~> Simplifier.add_cong
4167 delcongs ~> Simplifier.del_cong
4168 setmksimps ~> Simplifier.set_mksimps
4169 setmkcong ~> Simplifier.set_mkcong
4170 setmksym ~> Simplifier.set_mksym
4171 setmkeqTrue ~> Simplifier.set_mkeqTrue
4172 settermless ~> Simplifier.set_termless
4173 setsubgoaler ~> Simplifier.set_subgoaler
4174 addsplits ~> Splitter.add_split
4175 delsplits ~> Splitter.del_split
4180 * USER_HOME settings variable points to cross-platform user home
4181 directory, which coincides with HOME on POSIX systems only. Likewise,
4182 the Isabelle path specification "~" now expands to $USER_HOME, instead
4183 of former $HOME. A different default for USER_HOME may be set
4184 explicitly in shell environment, before Isabelle settings are
4185 evaluated. Minor INCOMPATIBILITY: need to adapt Isabelle path where
4186 the generic user home was intended.
4188 * ISABELLE_HOME_WINDOWS refers to ISABELLE_HOME in windows file name
4189 notation, which is useful for the jEdit file browser, for example.
4191 * ISABELLE_JDK_HOME settings variable points to JDK with javac and jar
4196 New in Isabelle2011-1 (October 2011)
4197 ------------------------------------
4201 * Improved Isabelle/jEdit Prover IDE (PIDE), which can be invoked as
4202 "isabelle jedit" or "ISABELLE_HOME/Isabelle" on the command line.
4204 - Management of multiple theory files directly from the editor
4205 buffer store -- bypassing the file-system (no requirement to save
4206 files for checking).
4208 - Markup of formal entities within the text buffer, with semantic
4209 highlighting, tooltips and hyperlinks to jump to defining source
4212 - Improved text rendering, with sub/superscripts in the source
4213 buffer (including support for copy/paste wrt. output panel, HTML
4214 theory output and other non-Isabelle text boxes).
4216 - Refined scheduling of proof checking and printing of results,
4217 based on interactive editor view. (Note: jEdit folding and
4218 narrowing allows to restrict buffer perspectives explicitly.)
4220 - Reduced CPU performance requirements, usable on machines with few
4223 - Reduced memory requirements due to pruning of unused document
4224 versions (garbage collection).
4226 See also ~~/src/Tools/jEdit/README.html for further information,
4227 including some remaining limitations.
4229 * Theory loader: source files are exclusively located via the master
4230 directory of each theory node (where the .thy file itself resides).
4231 The global load path (such as src/HOL/Library) has been discontinued.
4232 Note that the path element ~~ may be used to reference theories in the
4233 Isabelle home folder -- for instance, "~~/src/HOL/Library/FuncSet".
4236 * Theory loader: source files are identified by content via SHA1
4237 digests. Discontinued former path/modtime identification and optional
4238 ISABELLE_FILE_IDENT plugin scripts.
4240 * Parallelization of nested Isar proofs is subject to
4241 Goal.parallel_proofs_threshold (default 100). See also isabelle
4244 * Name space: former unsynchronized references are now proper
4245 configuration options, with more conventional names:
4247 long_names ~> names_long
4248 short_names ~> names_short
4249 unique_names ~> names_unique
4251 Minor INCOMPATIBILITY, need to declare options in context like this:
4253 declare [[names_unique = false]]
4255 * Literal facts `prop` may contain dummy patterns, e.g. `_ = _`. Note
4256 that the result needs to be unique, which means fact specifications
4257 may have to be refined after enriching a proof context.
4259 * Attribute "case_names" has been refined: the assumptions in each case
4260 can be named now by following the case name with [name1 name2 ...].
4262 * Isabelle/Isar reference manual has been updated and extended:
4263 - "Synopsis" provides a catalog of main Isar language concepts.
4264 - Formal references in syntax diagrams, via @{rail} antiquotation.
4265 - Updated material from classic "ref" manual, notably about
4266 "Classical Reasoner".
4271 * Class bot and top require underlying partial order rather than
4272 preorder: uniqueness of bot and top is guaranteed. INCOMPATIBILITY.
4274 * Class complete_lattice: generalized a couple of lemmas from sets;
4275 generalized theorems INF_cong and SUP_cong. New type classes for
4276 complete boolean algebras and complete linear orders. Lemmas
4277 Inf_less_iff, less_Sup_iff, INF_less_iff, less_SUP_iff now reside in
4278 class complete_linorder.
4280 Changed proposition of lemmas Inf_bool_def, Sup_bool_def, Inf_fun_def,
4281 Sup_fun_def, Inf_apply, Sup_apply.
4283 Removed redundant lemmas (the right hand side gives hints how to
4284 replace them for (metis ...), or (simp only: ...) proofs):
4286 Inf_singleton ~> Inf_insert [where A="{}", unfolded Inf_empty inf_top_right]
4287 Sup_singleton ~> Sup_insert [where A="{}", unfolded Sup_empty sup_bot_right]
4288 Inf_binary ~> Inf_insert, Inf_empty, and inf_top_right
4289 Sup_binary ~> Sup_insert, Sup_empty, and sup_bot_right
4290 Int_eq_Inter ~> Inf_insert, Inf_empty, and inf_top_right
4291 Un_eq_Union ~> Sup_insert, Sup_empty, and sup_bot_right
4292 Inter_def ~> INF_def, image_def
4293 Union_def ~> SUP_def, image_def
4294 INT_eq ~> INF_def, and image_def
4295 UN_eq ~> SUP_def, and image_def
4296 INF_subset ~> INF_superset_mono [OF _ order_refl]
4298 More consistent and comprehensive names:
4300 INTER_eq_Inter_image ~> INF_def
4301 UNION_eq_Union_image ~> SUP_def
4304 INF_leI ~> INF_lower
4305 INF_leI2 ~> INF_lower2
4306 le_INFI ~> INF_greatest
4307 le_SUPI ~> SUP_upper
4308 le_SUPI2 ~> SUP_upper2
4309 SUP_leI ~> SUP_least
4310 INFI_bool_eq ~> INF_bool_eq
4311 SUPR_bool_eq ~> SUP_bool_eq
4312 INFI_apply ~> INF_apply
4313 SUPR_apply ~> SUP_apply
4314 INTER_def ~> INTER_eq
4315 UNION_def ~> UNION_eq
4319 * Renamed theory Complete_Lattice to Complete_Lattices.
4322 * Theory Complete_Lattices: lemmas Inf_eq_top_iff, INF_eq_top_iff,
4323 INF_image, Inf_insert, INF_top, Inf_top_conv, INF_top_conv, SUP_bot,
4324 Sup_bot_conv, SUP_bot_conv, Sup_eq_top_iff, SUP_eq_top_iff, SUP_image,
4325 Sup_insert are now declared as [simp]. INCOMPATIBILITY.
4327 * Theory Lattice: lemmas compl_inf_bot, compl_le_comp_iff,
4328 compl_sup_top, inf_idem, inf_left_idem, inf_sup_absorb, sup_idem,
4329 sup_inf_absob, sup_left_idem are now declared as [simp]. Minor
4332 * Added syntactic classes "inf" and "sup" for the respective
4333 constants. INCOMPATIBILITY: Changes in the argument order of the
4334 (mostly internal) locale predicates for some derived classes.
4336 * Theorem collections ball_simps and bex_simps do not contain theorems
4337 referring to UNION any longer; these have been moved to collection
4338 UN_ball_bex_simps. INCOMPATIBILITY.
4340 * Theory Archimedean_Field: floor now is defined as parameter of a
4341 separate type class floor_ceiling.
4343 * Theory Finite_Set: more coherent development of fold_set locales:
4345 locale fun_left_comm ~> locale comp_fun_commute
4346 locale fun_left_comm_idem ~> locale comp_fun_idem
4348 Both use point-free characterization; interpretation proofs may need
4349 adjustment. INCOMPATIBILITY.
4351 * Theory Limits: Type "'a net" has been renamed to "'a filter", in
4352 accordance with standard mathematical terminology. INCOMPATIBILITY.
4354 * Theory Complex_Main: The locale interpretations for the
4355 bounded_linear and bounded_bilinear locales have been removed, in
4356 order to reduce the number of duplicate lemmas. Users must use the
4357 original names for distributivity theorems, potential INCOMPATIBILITY.
4359 divide.add ~> add_divide_distrib
4360 divide.diff ~> diff_divide_distrib
4361 divide.setsum ~> setsum_divide_distrib
4362 mult.add_right ~> right_distrib
4363 mult.diff_right ~> right_diff_distrib
4364 mult_right.setsum ~> setsum_right_distrib
4365 mult_left.diff ~> left_diff_distrib
4367 * Theory Complex_Main: Several redundant theorems have been removed or
4368 replaced by more general versions. INCOMPATIBILITY.
4370 real_diff_def ~> minus_real_def
4371 real_divide_def ~> divide_real_def
4372 real_less_def ~> less_le
4373 real_abs_def ~> abs_real_def
4374 real_sgn_def ~> sgn_real_def
4375 real_mult_commute ~> mult_commute
4376 real_mult_assoc ~> mult_assoc
4377 real_mult_1 ~> mult_1_left
4378 real_add_mult_distrib ~> left_distrib
4379 real_zero_not_eq_one ~> zero_neq_one
4380 real_mult_inverse_left ~> left_inverse
4381 INVERSE_ZERO ~> inverse_zero
4382 real_le_refl ~> order_refl
4383 real_le_antisym ~> order_antisym
4384 real_le_trans ~> order_trans
4385 real_le_linear ~> linear
4386 real_le_eq_diff ~> le_iff_diff_le_0
4387 real_add_left_mono ~> add_left_mono
4388 real_mult_order ~> mult_pos_pos
4389 real_mult_less_mono2 ~> mult_strict_left_mono
4390 real_of_int_real_of_nat ~> real_of_int_of_nat_eq
4391 real_0_le_divide_iff ~> zero_le_divide_iff
4392 realpow_two_disj ~> power2_eq_iff
4393 real_squared_diff_one_factored ~> square_diff_one_factored
4394 realpow_two_diff ~> square_diff_square_factored
4395 reals_complete2 ~> complete_real
4396 real_sum_squared_expand ~> power2_sum
4397 exp_ln_eq ~> ln_unique
4399 expi_zero ~> exp_zero
4400 lemma_DERIV_subst ~> DERIV_cong
4401 LIMSEQ_Zfun_iff ~> tendsto_Zfun_iff
4402 LIMSEQ_const ~> tendsto_const
4403 LIMSEQ_norm ~> tendsto_norm
4404 LIMSEQ_add ~> tendsto_add
4405 LIMSEQ_minus ~> tendsto_minus
4406 LIMSEQ_minus_cancel ~> tendsto_minus_cancel
4407 LIMSEQ_diff ~> tendsto_diff
4408 bounded_linear.LIMSEQ ~> bounded_linear.tendsto
4409 bounded_bilinear.LIMSEQ ~> bounded_bilinear.tendsto
4410 LIMSEQ_mult ~> tendsto_mult
4411 LIMSEQ_inverse ~> tendsto_inverse
4412 LIMSEQ_divide ~> tendsto_divide
4413 LIMSEQ_pow ~> tendsto_power
4414 LIMSEQ_setsum ~> tendsto_setsum
4415 LIMSEQ_setprod ~> tendsto_setprod
4416 LIMSEQ_norm_zero ~> tendsto_norm_zero_iff
4417 LIMSEQ_rabs_zero ~> tendsto_rabs_zero_iff
4418 LIMSEQ_imp_rabs ~> tendsto_rabs
4419 LIMSEQ_add_minus ~> tendsto_add [OF _ tendsto_minus]
4420 LIMSEQ_add_const ~> tendsto_add [OF _ tendsto_const]
4421 LIMSEQ_diff_const ~> tendsto_diff [OF _ tendsto_const]
4422 LIMSEQ_Complex ~> tendsto_Complex
4423 LIM_ident ~> tendsto_ident_at
4424 LIM_const ~> tendsto_const
4425 LIM_add ~> tendsto_add
4426 LIM_add_zero ~> tendsto_add_zero
4427 LIM_minus ~> tendsto_minus
4428 LIM_diff ~> tendsto_diff
4429 LIM_norm ~> tendsto_norm
4430 LIM_norm_zero ~> tendsto_norm_zero
4431 LIM_norm_zero_cancel ~> tendsto_norm_zero_cancel
4432 LIM_norm_zero_iff ~> tendsto_norm_zero_iff
4433 LIM_rabs ~> tendsto_rabs
4434 LIM_rabs_zero ~> tendsto_rabs_zero
4435 LIM_rabs_zero_cancel ~> tendsto_rabs_zero_cancel
4436 LIM_rabs_zero_iff ~> tendsto_rabs_zero_iff
4437 LIM_compose ~> tendsto_compose
4438 LIM_mult ~> tendsto_mult
4439 LIM_scaleR ~> tendsto_scaleR
4440 LIM_of_real ~> tendsto_of_real
4441 LIM_power ~> tendsto_power
4442 LIM_inverse ~> tendsto_inverse
4443 LIM_sgn ~> tendsto_sgn
4444 isCont_LIM_compose ~> isCont_tendsto_compose
4445 bounded_linear.LIM ~> bounded_linear.tendsto
4446 bounded_linear.LIM_zero ~> bounded_linear.tendsto_zero
4447 bounded_bilinear.LIM ~> bounded_bilinear.tendsto
4448 bounded_bilinear.LIM_prod_zero ~> bounded_bilinear.tendsto_zero
4449 bounded_bilinear.LIM_left_zero ~> bounded_bilinear.tendsto_left_zero
4450 bounded_bilinear.LIM_right_zero ~> bounded_bilinear.tendsto_right_zero
4451 LIM_inverse_fun ~> tendsto_inverse [OF tendsto_ident_at]
4453 * Theory Complex_Main: The definition of infinite series was
4454 generalized. Now it is defined on the type class {topological_space,
4455 comm_monoid_add}. Hence it is useable also for extended real numbers.
4457 * Theory Complex_Main: The complex exponential function "expi" is now
4458 a type-constrained abbreviation for "exp :: complex => complex"; thus
4459 several polymorphic lemmas about "exp" are now applicable to "expi".
4463 - Theory Library/Code_Char_ord provides native ordering of
4464 characters in the target language.
4466 - Commands code_module and code_library are legacy, use export_code
4469 - Method "evaluation" is legacy, use method "eval" instead.
4471 - Legacy evaluator "SML" is deactivated by default. May be
4472 reactivated by the following theory command:
4474 setup {* Value.add_evaluator ("SML", Codegen.eval_term) *}
4476 * Declare ext [intro] by default. Rare INCOMPATIBILITY.
4478 * New proof method "induction" that gives induction hypotheses the
4479 name "IH", thus distinguishing them from further hypotheses that come
4480 from rule induction. The latter are still called "hyps". Method
4481 "induction" is a thin wrapper around "induct" and follows the same
4484 * Method "fastsimp" has been renamed to "fastforce", but "fastsimp" is
4485 still available as a legacy feature for some time.
4488 - Added "need" and "total_consts" options.
4489 - Reintroduced "show_skolems" option by popular demand.
4490 - Renamed attribute: nitpick_def ~> nitpick_unfold.
4494 - Use quasi-sound (and efficient) translations by default.
4495 - Added support for the following provers: E-ToFoF, LEO-II,
4496 Satallax, SNARK, Waldmeister, and Z3 with TPTP syntax.
4497 - Automatically preplay and minimize proofs before showing them if
4498 this can be done within reasonable time.
4499 - sledgehammer available_provers ~> sledgehammer supported_provers.
4501 - Added "preplay_timeout", "slicing", "type_enc", "sound",
4502 "max_mono_iters", and "max_new_mono_instances" options.
4503 - Removed "explicit_apply" and "full_types" options as well as "Full
4504 Types" Proof General menu item. INCOMPATIBILITY.
4507 - Removed "metisF" -- use "metis" instead. INCOMPATIBILITY.
4508 - Obsoleted "metisFT" -- use "metis (full_types)" instead.
4512 - Renamed 'try_methods' and added "simp:", "intro:", "dest:", and
4513 "elim:" options. INCOMPATIBILITY.
4514 - Introduced 'try' that not only runs 'try_methods' but also
4515 'solve_direct', 'sledgehammer', 'quickcheck', and 'nitpick'.
4518 - Added "eval" option to evaluate terms for the found counterexample
4519 (currently only supported by the default (exhaustive) tester).
4520 - Added post-processing of terms to obtain readable counterexamples
4521 (currently only supported by the default (exhaustive) tester).
4522 - New counterexample generator quickcheck[narrowing] enables
4523 narrowing-based testing. Requires the Glasgow Haskell compiler
4524 with its installation location defined in the Isabelle settings
4525 environment as ISABELLE_GHC.
4526 - Removed quickcheck tester "SML" based on the SML code generator
4527 (formly in HOL/Library).
4529 * Function package: discontinued option "tailrec". INCOMPATIBILITY,
4530 use 'partial_function' instead.
4532 * Theory Library/Extended_Reals replaces now the positive extended
4533 reals found in probability theory. This file is extended by
4534 Multivariate_Analysis/Extended_Real_Limits.
4536 * Theory Library/Old_Recdef: old 'recdef' package has been moved here,
4537 from where it must be imported explicitly if it is really required.
4540 * Theory Library/Wfrec: well-founded recursion combinator "wfrec" has
4541 been moved here. INCOMPATIBILITY.
4543 * Theory Library/Saturated provides type of numbers with saturated
4546 * Theory Library/Product_Lattice defines a pointwise ordering for the
4547 product type 'a * 'b, and provides instance proofs for various order
4548 and lattice type classes.
4550 * Theory Library/Countable now provides the "countable_datatype" proof
4551 method for proving "countable" class instances for datatypes.
4553 * Theory Library/Cset_Monad allows do notation for computable sets
4554 (cset) via the generic monad ad-hoc overloading facility.
4556 * Library: Theories of common data structures are split into theories
4557 for implementation, an invariant-ensuring type, and connection to an
4558 abstract type. INCOMPATIBILITY.
4560 - RBT is split into RBT and RBT_Mapping.
4561 - AssocList is split and renamed into AList and AList_Mapping.
4562 - DList is split into DList_Impl, DList, and DList_Cset.
4563 - Cset is split into Cset and List_Cset.
4565 * Theory Library/Nat_Infinity has been renamed to
4566 Library/Extended_Nat, with name changes of the following types and
4569 type inat ~> type enat
4571 Infty ~> infinity (overloaded)
4575 Every theorem name containing "inat", "Fin", "Infty", or "iSuc" has
4576 been renamed accordingly. INCOMPATIBILITY.
4578 * Session Multivariate_Analysis: The euclidean_space type class now
4579 fixes a constant "Basis :: 'a set" consisting of the standard
4580 orthonormal basis for the type. Users now have the option of
4581 quantifying over this set instead of using the "basis" function, e.g.
4582 "ALL x:Basis. P x" vs "ALL i<DIM('a). P (basis i)".
4584 * Session Multivariate_Analysis: Type "('a, 'b) cart" has been renamed
4585 to "('a, 'b) vec" (the syntax "'a ^ 'b" remains unaffected). Constants
4586 "Cart_nth" and "Cart_lambda" have been respectively renamed to
4587 "vec_nth" and "vec_lambda"; theorems mentioning those names have
4588 changed to match. Definition theorems for overloaded constants now use
4589 the standard "foo_vec_def" naming scheme. A few other theorems have
4590 been renamed as follows (INCOMPATIBILITY):
4592 Cart_eq ~> vec_eq_iff
4593 dist_nth_le_cart ~> dist_vec_nth_le
4594 tendsto_vector ~> vec_tendstoI
4595 Cauchy_vector ~> vec_CauchyI
4597 * Session Multivariate_Analysis: Several duplicate theorems have been
4598 removed, and other theorems have been renamed or replaced with more
4599 general versions. INCOMPATIBILITY.
4601 finite_choice ~> finite_set_choice
4602 eventually_conjI ~> eventually_conj
4603 eventually_and ~> eventually_conj_iff
4604 eventually_false ~> eventually_False
4605 setsum_norm ~> norm_setsum
4606 Lim_sequentially ~> LIMSEQ_def
4607 Lim_ident_at ~> LIM_ident
4608 Lim_const ~> tendsto_const
4609 Lim_cmul ~> tendsto_scaleR [OF tendsto_const]
4610 Lim_neg ~> tendsto_minus
4611 Lim_add ~> tendsto_add
4612 Lim_sub ~> tendsto_diff
4613 Lim_mul ~> tendsto_scaleR
4614 Lim_vmul ~> tendsto_scaleR [OF _ tendsto_const]
4615 Lim_null_norm ~> tendsto_norm_zero_iff [symmetric]
4616 Lim_linear ~> bounded_linear.tendsto
4617 Lim_component ~> tendsto_euclidean_component
4618 Lim_component_cart ~> tendsto_vec_nth
4619 Lim_inner ~> tendsto_inner [OF tendsto_const]
4620 dot_lsum ~> inner_setsum_left
4621 dot_rsum ~> inner_setsum_right
4622 continuous_cmul ~> continuous_scaleR [OF continuous_const]
4623 continuous_neg ~> continuous_minus
4624 continuous_sub ~> continuous_diff
4625 continuous_vmul ~> continuous_scaleR [OF _ continuous_const]
4626 continuous_mul ~> continuous_scaleR
4627 continuous_inv ~> continuous_inverse
4628 continuous_at_within_inv ~> continuous_at_within_inverse
4629 continuous_at_inv ~> continuous_at_inverse
4630 continuous_at_norm ~> continuous_norm [OF continuous_at_id]
4631 continuous_at_infnorm ~> continuous_infnorm [OF continuous_at_id]
4632 continuous_at_component ~> continuous_component [OF continuous_at_id]
4633 continuous_on_neg ~> continuous_on_minus
4634 continuous_on_sub ~> continuous_on_diff
4635 continuous_on_cmul ~> continuous_on_scaleR [OF continuous_on_const]
4636 continuous_on_vmul ~> continuous_on_scaleR [OF _ continuous_on_const]
4637 continuous_on_mul ~> continuous_on_scaleR
4638 continuous_on_mul_real ~> continuous_on_mult
4639 continuous_on_inner ~> continuous_on_inner [OF continuous_on_const]
4640 continuous_on_norm ~> continuous_on_norm [OF continuous_on_id]
4641 continuous_on_inverse ~> continuous_on_inv
4642 uniformly_continuous_on_neg ~> uniformly_continuous_on_minus
4643 uniformly_continuous_on_sub ~> uniformly_continuous_on_diff
4644 subset_interior ~> interior_mono
4645 subset_closure ~> closure_mono
4646 closure_univ ~> closure_UNIV
4647 real_arch_lt ~> reals_Archimedean2
4648 real_arch ~> reals_Archimedean3
4649 real_abs_norm ~> abs_norm_cancel
4650 real_abs_sub_norm ~> norm_triangle_ineq3
4651 norm_cauchy_schwarz_abs ~> Cauchy_Schwarz_ineq2
4653 * Session HOL-Probability:
4654 - Caratheodory's extension lemma is now proved for ring_of_sets.
4655 - Infinite products of probability measures are now available.
4656 - Sigma closure is independent, if the generator is independent
4657 - Use extended reals instead of positive extended
4658 reals. INCOMPATIBILITY.
4660 * Session HOLCF: Discontinued legacy theorem names, INCOMPATIBILITY.
4662 expand_fun_below ~> fun_below_iff
4663 below_fun_ext ~> fun_belowI
4664 expand_cfun_eq ~> cfun_eq_iff
4665 ext_cfun ~> cfun_eqI
4666 expand_cfun_below ~> cfun_below_iff
4667 below_cfun_ext ~> cfun_belowI
4668 monofun_fun_fun ~> fun_belowD
4669 monofun_fun_arg ~> monofunE
4670 monofun_lub_fun ~> adm_monofun [THEN admD]
4671 cont_lub_fun ~> adm_cont [THEN admD]
4672 cont2cont_Rep_CFun ~> cont2cont_APP
4673 cont_Rep_CFun_app ~> cont_APP_app
4674 cont_Rep_CFun_app_app ~> cont_APP_app_app
4675 cont_cfun_fun ~> cont_Rep_cfun1 [THEN contE]
4676 cont_cfun_arg ~> cont_Rep_cfun2 [THEN contE]
4677 contlub_cfun ~> lub_APP [symmetric]
4678 contlub_LAM ~> lub_LAM [symmetric]
4681 lift_distinct1 ~> lift.distinct(1)
4682 lift_distinct2 ~> lift.distinct(2)
4683 Def_not_UU ~> lift.distinct(2)
4684 Def_inject ~> lift.inject
4685 below_UU_iff ~> below_bottom_iff
4686 eq_UU_iff ~> eq_bottom_iff
4689 *** Document preparation ***
4691 * Antiquotation @{rail} layouts railroad syntax diagrams, see also
4692 isar-ref manual, both for description and actual application of the
4695 * Antiquotation @{value} evaluates the given term and presents its
4698 * Antiquotations: term style "isub" provides ad-hoc conversion of
4699 variables x1, y23 into subscripted form x\<^isub>1,
4700 y\<^isub>2\<^isub>3.
4702 * Predefined LaTeX macros for Isabelle symbols \<bind> and \<then>
4703 (e.g. see ~~/src/HOL/Library/Monad_Syntax.thy).
4705 * Localized \isabellestyle switch can be used within blocks or groups
4708 \isabellestyle{it} %preferred default
4709 {\isabellestylett @{text "typewriter stuff"}}
4711 * Discontinued special treatment of hard tabulators. Implicit
4712 tab-width is now defined as 1. Potential INCOMPATIBILITY for visual
4718 * The inner syntax of sort/type/term/prop supports inlined YXML
4719 representations within quoted string tokens. By encoding logical
4720 entities via Term_XML (in ML or Scala) concrete syntax can be
4721 bypassed, which is particularly useful for producing bits of text
4722 under external program control.
4724 * Antiquotations for ML and document preparation are managed as theory
4725 data, which requires explicit setup.
4727 * Isabelle_Process.is_active allows tools to check if the official
4728 process wrapper is running (Isabelle/Scala/jEdit) or the old TTY loop
4729 (better known as Proof General).
4731 * Structure Proof_Context follows standard naming scheme. Old
4732 ProofContext is still available for some time as legacy alias.
4734 * Structure Timing provides various operations for timing; supersedes
4735 former start_timing/end_timing etc.
4737 * Path.print is the official way to show file-system paths to users
4738 (including quotes etc.).
4740 * Inner syntax: identifiers in parse trees of generic categories
4741 "logic", "aprop", "idt" etc. carry position information (disguised as
4742 type constraints). Occasional INCOMPATIBILITY with non-compliant
4743 translations that choke on unexpected type constraints. Positions can
4744 be stripped in ML translations via Syntax.strip_positions /
4745 Syntax.strip_positions_ast, or via the syntax constant
4746 "_strip_positions" within parse trees. As last resort, positions can
4747 be disabled via the configuration option Syntax.positions, which is
4748 called "syntax_positions" in Isar attribute syntax.
4750 * Discontinued special status of various ML structures that contribute
4751 to structure Syntax (Ast, Lexicon, Mixfix, Parser, Printer etc.): less
4752 pervasive content, no inclusion in structure Syntax. INCOMPATIBILITY,
4753 refer directly to Ast.Constant, Lexicon.is_identifier,
4754 Syntax_Trans.mk_binder_tr etc.
4756 * Typed print translation: discontinued show_sorts argument, which is
4757 already available via context of "advanced" translation.
4759 * Refined PARALLEL_GOALS tactical: degrades gracefully for schematic
4760 goal states; body tactic needs to address all subgoals uniformly.
4762 * Slightly more special eq_list/eq_set, with shortcut involving
4763 pointer equality (assumes that eq relation is reflexive).
4765 * Classical tactics use proper Proof.context instead of historic types
4766 claset/clasimpset. Old-style declarations like addIs, addEs, addDs
4767 operate directly on Proof.context. Raw type claset retains its use as
4768 snapshot of the classical context, which can be recovered via
4769 (put_claset HOL_cs) etc. Type clasimpset has been discontinued.
4770 INCOMPATIBILITY, classical tactics and derived proof methods require
4771 proper Proof.context.
4776 * Discontinued support for Poly/ML 5.2, which was the last version
4777 without proper multithreading and TimeLimit implementation.
4779 * Discontinued old lib/scripts/polyml-platform, which has been
4780 obsolete since Isabelle2009-2.
4782 * Various optional external tools are referenced more robustly and
4783 uniformly by explicit Isabelle settings as follows:
4785 ISABELLE_CSDP (formerly CSDP_EXE)
4786 ISABELLE_GHC (formerly EXEC_GHC or GHC_PATH)
4787 ISABELLE_OCAML (formerly EXEC_OCAML)
4788 ISABELLE_SWIPL (formerly EXEC_SWIPL)
4789 ISABELLE_YAP (formerly EXEC_YAP)
4791 Note that automated detection from the file-system or search path has
4792 been discontinued. INCOMPATIBILITY.
4794 * Scala layer provides JVM method invocation service for static
4795 methods of type (String)String, see Invoke_Scala.method in ML. For
4798 Invoke_Scala.method "java.lang.System.getProperty" "java.home"
4800 Together with YXML.string_of_body/parse_body and XML.Encode/Decode
4801 this allows to pass structured values between ML and Scala.
4803 * The IsabelleText fonts includes some further glyphs to support the
4804 Prover IDE. Potential INCOMPATIBILITY: users who happen to have
4805 installed a local copy (which is normally *not* required) need to
4806 delete or update it from ~~/lib/fonts/.
4810 New in Isabelle2011 (January 2011)
4811 ----------------------------------
4815 * Experimental Prover IDE based on Isabelle/Scala and jEdit (see
4816 src/Tools/jEdit). This also serves as IDE for Isabelle/ML, with
4817 useful tooltips and hyperlinks produced from its static analysis. The
4818 bundled component provides an executable Isabelle tool that can be run
4821 Isabelle2011/bin/isabelle jedit
4823 * Significantly improved Isabelle/Isar implementation manual.
4825 * System settings: ISABELLE_HOME_USER now includes ISABELLE_IDENTIFIER
4826 (and thus refers to something like $HOME/.isabelle/Isabelle2011),
4827 while the default heap location within that directory lacks that extra
4828 suffix. This isolates multiple Isabelle installations from each
4829 other, avoiding problems with old settings in new versions.
4830 INCOMPATIBILITY, need to copy/upgrade old user settings manually.
4832 * Source files are always encoded as UTF-8, instead of old-fashioned
4833 ISO-Latin-1. INCOMPATIBILITY. Isabelle LaTeX documents might require
4834 the following package declarations:
4836 \usepackage[utf8]{inputenc}
4837 \usepackage{textcomp}
4839 * Explicit treatment of UTF-8 sequences as Isabelle symbols, such that
4840 a Unicode character is treated as a single symbol, not a sequence of
4841 non-ASCII bytes as before. Since Isabelle/ML string literals may
4842 contain symbols without further backslash escapes, Unicode can now be
4843 used here as well. Recall that Symbol.explode in ML provides a
4844 consistent view on symbols, while raw explode (or String.explode)
4845 merely give a byte-oriented representation.
4847 * Theory loader: source files are primarily located via the master
4848 directory of each theory node (where the .thy file itself resides).
4849 The global load path is still partially available as legacy feature.
4850 Minor INCOMPATIBILITY due to subtle change in file lookup: use
4851 explicit paths, relatively to the theory.
4853 * Special treatment of ML file names has been discontinued.
4854 Historically, optional extensions .ML or .sml were added on demand --
4855 at the cost of clarity of file dependencies. Recall that Isabelle/ML
4856 files exclusively use the .ML extension. Minor INCOMPATIBILITY.
4858 * Various options that affect pretty printing etc. are now properly
4859 handled within the context via configuration options, instead of
4860 unsynchronized references or print modes. There are both ML Config.T
4861 entities and Isar declaration attributes to access these.
4863 ML (Config.T) Isar (attribute)
4865 eta_contract eta_contract
4866 show_brackets show_brackets
4867 show_sorts show_sorts
4868 show_types show_types
4869 show_question_marks show_question_marks
4870 show_consts show_consts
4871 show_abbrevs show_abbrevs
4873 Syntax.ast_trace syntax_ast_trace
4874 Syntax.ast_stat syntax_ast_stat
4875 Syntax.ambiguity_level syntax_ambiguity_level
4877 Goal_Display.goals_limit goals_limit
4878 Goal_Display.show_main_goal show_main_goal
4880 Method.rule_trace rule_trace
4882 Thy_Output.display thy_output_display
4883 Thy_Output.quotes thy_output_quotes
4884 Thy_Output.indent thy_output_indent
4885 Thy_Output.source thy_output_source
4886 Thy_Output.break thy_output_break
4888 Note that corresponding "..._default" references in ML may only be
4889 changed globally at the ROOT session setup, but *not* within a theory.
4890 The option "show_abbrevs" supersedes the former print mode
4891 "no_abbrevs" with inverted meaning.
4893 * More systematic naming of some configuration options.
4896 trace_simp ~> simp_trace
4897 debug_simp ~> simp_debug
4899 * Support for real valued configuration options, using simplistic
4900 floating-point notation that coincides with the inner syntax for
4903 * Support for real valued preferences (with approximative PGIP type):
4904 front-ends need to accept "pgint" values in float notation.
4907 * The IsabelleText font now includes Cyrillic, Hebrew, Arabic from
4910 * Discontinued support for Poly/ML 5.0 and 5.1 versions.
4915 * Command 'type_synonym' (with single argument) replaces somewhat
4916 outdated 'types', which is still available as legacy feature for some
4919 * Command 'nonterminal' (with 'and' separated list of arguments)
4920 replaces somewhat outdated 'nonterminals'. INCOMPATIBILITY.
4922 * Command 'notepad' replaces former 'example_proof' for
4923 experimentation in Isar without any result. INCOMPATIBILITY.
4925 * Locale interpretation commands 'interpret' and 'sublocale' accept
4926 lists of equations to map definitions in a locale to appropriate
4927 entities in the context of the interpretation. The 'interpretation'
4928 command already provided this functionality.
4930 * Diagnostic command 'print_dependencies' prints the locale instances
4931 that would be activated if the specified expression was interpreted in
4932 the current context. Variant "print_dependencies!" assumes a context
4933 without interpretations.
4935 * Diagnostic command 'print_interps' prints interpretations in proofs
4936 in addition to interpretations in theories.
4938 * Discontinued obsolete 'global' and 'local' commands to manipulate
4939 the theory name space. Rare INCOMPATIBILITY. The ML functions
4940 Sign.root_path and Sign.local_path may be applied directly where this
4941 feature is still required for historical reasons.
4943 * Discontinued obsolete 'constdefs' command. INCOMPATIBILITY, use
4944 'definition' instead.
4946 * The "prems" fact, which refers to the accidental collection of
4947 foundational premises in the context, is now explicitly marked as
4948 legacy feature and will be discontinued soon. Consider using "assms"
4949 of the head statement or reference facts by explicit names.
4951 * Document antiquotations @{class} and @{type} print classes and type
4954 * Document antiquotation @{file} checks file/directory entries within
4955 the local file system.
4960 * Coercive subtyping: functions can be declared as coercions and type
4961 inference will add them as necessary upon input of a term. Theory
4962 Complex_Main declares real :: nat => real and real :: int => real as
4963 coercions. A coercion function f is declared like this:
4965 declare [[coercion f]]
4967 To lift coercions through type constructors (e.g. from nat => real to
4968 nat list => real list), map functions can be declared, e.g.
4970 declare [[coercion_map map]]
4972 Currently coercion inference is activated only in theories including
4973 real numbers, i.e. descendants of Complex_Main. This is controlled by
4974 the configuration option "coercion_enabled", e.g. it can be enabled in
4975 other theories like this:
4977 declare [[coercion_enabled]]
4979 * Command 'partial_function' provides basic support for recursive
4980 function definitions over complete partial orders. Concrete instances
4981 are provided for i) the option type, ii) tail recursion on arbitrary
4982 types, and iii) the heap monad of Imperative_HOL. See
4983 src/HOL/ex/Fundefs.thy and src/HOL/Imperative_HOL/ex/Linked_Lists.thy
4986 * Function package: f.psimps rules are no longer implicitly declared
4987 as [simp]. INCOMPATIBILITY.
4989 * Datatype package: theorems generated for executable equality (class
4990 "eq") carry proper names and are treated as default code equations.
4992 * Inductive package: now offers command 'inductive_simps' to
4993 automatically derive instantiated and simplified equations for
4994 inductive predicates, similar to 'inductive_cases'.
4996 * Command 'enriched_type' allows to register properties of the
4997 functorial structure of types.
4999 * Improved infrastructure for term evaluation using code generator
5000 techniques, in particular static evaluation conversions.
5002 * Code generator: Scala (2.8 or higher) has been added to the target
5005 * Code generator: globbing constant expressions "*" and "Theory.*"
5006 have been replaced by the more idiomatic "_" and "Theory._".
5009 * Code generator: export_code without explicit file declaration prints
5010 to standard output. INCOMPATIBILITY.
5012 * Code generator: do not print function definitions for case
5013 combinators any longer.
5015 * Code generator: simplification with rules determined with
5016 src/Tools/Code/code_simp.ML and method "code_simp".
5018 * Code generator for records: more idiomatic representation of record
5019 types. Warning: records are not covered by ancient SML code
5020 generation any longer. INCOMPATIBILITY. In cases of need, a suitable
5021 rep_datatype declaration helps to succeed then:
5025 rep_datatype foo_ext ...
5027 * Records: logical foundation type for records does not carry a
5028 '_type' suffix any longer (obsolete due to authentic syntax).
5031 * Quickcheck now by default uses exhaustive testing instead of random
5032 testing. Random testing can be invoked by "quickcheck [random]",
5033 exhaustive testing by "quickcheck [exhaustive]".
5035 * Quickcheck instantiates polymorphic types with small finite
5036 datatypes by default. This enables a simple execution mechanism to
5037 handle quantifiers and function equality over the finite datatypes.
5039 * Quickcheck random generator has been renamed from "code" to
5040 "random". INCOMPATIBILITY.
5042 * Quickcheck now has a configurable time limit which is set to 30
5043 seconds by default. This can be changed by adding [timeout = n] to the
5044 quickcheck command. The time limit for Auto Quickcheck is still set
5047 * Quickcheck in locales considers interpretations of that locale for
5048 counter example search.
5051 - Added "smt" and "remote_smt" provers based on the "smt" proof
5052 method. See the Sledgehammer manual for details ("isabelle doc
5055 sledgehammer atp_info ~> sledgehammer running_provers
5056 sledgehammer atp_kill ~> sledgehammer kill_provers
5057 sledgehammer available_atps ~> sledgehammer available_provers
5060 sledgehammer [atps = ...] ~> sledgehammer [provers = ...]
5061 sledgehammer [atp = ...] ~> sledgehammer [prover = ...]
5062 sledgehammer [timeout = 77 s] ~> sledgehammer [timeout = 77]
5063 (and "ms" and "min" are no longer supported)
5068 nitpick [timeout = 77 s] ~> nitpick [timeout = 77]
5069 nitpick [tac_timeout = 777 ms] ~> nitpick [tac_timeout = 0.777]
5071 - Added support for partial quotient types.
5072 - Added local versions of the "Nitpick.register_xxx" functions.
5073 - Added "whack" option.
5074 - Allow registration of quotient types as codatatypes.
5075 - Improved "merge_type_vars" option to merge more types.
5076 - Removed unsound "fast_descrs" option.
5077 - Added custom symmetry breaking for datatypes, making it possible to reach
5078 higher cardinalities.
5079 - Prevent the expansion of too large definitions.
5081 * Proof methods "metis" and "meson" now have configuration options
5082 "meson_trace", "metis_trace", and "metis_verbose" that can be enabled
5083 to diagnose these tools. E.g.
5085 using [[metis_trace = true]]
5087 * Auto Solve: Renamed "Auto Solve Direct". The tool is now available
5088 manually as command 'solve_direct'.
5090 * The default SMT solver Z3 must be enabled explicitly (due to
5091 licensing issues) by setting the environment variable
5092 Z3_NON_COMMERCIAL in etc/settings of the component, for example. For
5093 commercial applications, the SMT solver CVC3 is provided as fall-back;
5094 changing the SMT solver is done via the configuration option
5097 * Remote SMT solvers need to be referred to by the "remote_" prefix,
5098 i.e. "remote_cvc3" and "remote_z3".
5100 * Added basic SMT support for datatypes, records, and typedefs using
5101 the oracle mode (no proofs). Direct support of pairs has been dropped
5102 in exchange (pass theorems fst_conv snd_conv pair_collapse to the SMT
5103 support for a similar behavior). Minor INCOMPATIBILITY.
5105 * Changed SMT configuration options:
5107 z3_proofs ~> smt_oracle (with inverted meaning)
5108 z3_trace_assms ~> smt_trace_used_facts
5121 * Boogie output files (.b2i files) need to be declared in the theory
5124 * Simplification procedure "list_to_set_comprehension" rewrites list
5125 comprehensions applied to List.set to set comprehensions. Occasional
5126 INCOMPATIBILITY, may be deactivated like this:
5128 declare [[simproc del: list_to_set_comprehension]]
5130 * Removed old version of primrec package. INCOMPATIBILITY.
5132 * Removed simplifier congruence rule of "prod_case", as has for long
5133 been the case with "split". INCOMPATIBILITY.
5135 * String.literal is a type, but not a datatype. INCOMPATIBILITY.
5137 * Removed [split_format ... and ... and ...] version of
5138 [split_format]. Potential INCOMPATIBILITY.
5140 * Predicate "sorted" now defined inductively, with nice induction
5141 rules. INCOMPATIBILITY: former sorted.simps now named sorted_simps.
5143 * Constant "contents" renamed to "the_elem", to free the generic name
5144 contents for other uses. INCOMPATIBILITY.
5146 * Renamed class eq and constant eq (for code generation) to class
5147 equal and constant equal, plus renaming of related facts and various
5148 tuning. INCOMPATIBILITY.
5150 * Dropped type classes mult_mono and mult_mono1. INCOMPATIBILITY.
5152 * Removed output syntax "'a ~=> 'b" for "'a => 'b option".
5155 * Renamed theory Fset to Cset, type Fset.fset to Cset.set, in order to
5156 avoid confusion with finite sets. INCOMPATIBILITY.
5158 * Abandoned locales equiv, congruent and congruent2 for equivalence
5159 relations. INCOMPATIBILITY: use equivI rather than equiv_intro (same
5162 * Some previously unqualified names have been qualified:
5169 Trueprop ~> HOL.Trueprop
5174 op --> ~> HOL.implies
5186 Pair ~> Product_Type.Pair
5187 fst ~> Product_Type.fst
5188 snd ~> Product_Type.snd
5189 curry ~> Product_Type.curry
5191 Collect ~> Set.Collect
5195 * More canonical naming convention for some fundamental definitions:
5197 bot_bool_eq ~> bot_bool_def
5198 top_bool_eq ~> top_bool_def
5199 inf_bool_eq ~> inf_bool_def
5200 sup_bool_eq ~> sup_bool_def
5201 bot_fun_eq ~> bot_fun_def
5202 top_fun_eq ~> top_fun_def
5203 inf_fun_eq ~> inf_fun_def
5204 sup_fun_eq ~> sup_fun_def
5208 * More stylized fact names:
5210 expand_fun_eq ~> fun_eq_iff
5211 expand_set_eq ~> set_eq_iff
5213 nat_number ~> eval_nat_numeral
5217 * Refactoring of code-generation specific operations in theory List:
5223 mem_iff ~> member_def
5224 null_empty ~> null_def
5226 INCOMPATIBILITY. Note that these were not supposed to be used
5227 regularly unless for striking reasons; their main purpose was code
5230 Various operations from the Haskell prelude are used for generating
5233 * Term "bij f" is now an abbreviation of "bij_betw f UNIV UNIV". Term
5234 "surj f" is now an abbreviation of "range f = UNIV". The theorems
5235 bij_def and surj_def are unchanged. INCOMPATIBILITY.
5237 * Abolished some non-alphabetic type names: "prod" and "sum" replace
5238 "*" and "+" respectively. INCOMPATIBILITY.
5240 * Name "Plus" of disjoint sum operator "<+>" is now hidden. Write
5241 "Sum_Type.Plus" instead.
5243 * Constant "split" has been merged with constant "prod_case"; names of
5244 ML functions, facts etc. involving split have been retained so far,
5245 though. INCOMPATIBILITY.
5247 * Dropped old infix syntax "_ mem _" for List.member; use "_ : set _"
5248 instead. INCOMPATIBILITY.
5250 * Removed lemma "Option.is_none_none" which duplicates "is_none_def".
5253 * Former theory Library/Enum is now part of the HOL-Main image.
5254 INCOMPATIBILITY: all constants of the Enum theory now have to be
5255 referred to by its qualified name.
5258 nlists ~> Enum.nlists
5259 product ~> Enum.product
5261 * Theory Library/Monad_Syntax provides do-syntax for monad types.
5262 Syntax in Library/State_Monad has been changed to avoid ambiguities.
5265 * Theory Library/SetsAndFunctions has been split into
5266 Library/Function_Algebras and Library/Set_Algebras; canonical names
5267 for instance definitions for functions; various improvements.
5270 * Theory Library/Multiset provides stable quicksort implementation of
5273 * Theory Library/Multiset: renamed empty_idemp ~> empty_neutral.
5276 * Session Multivariate_Analysis: introduced a type class for euclidean
5277 space. Most theorems are now stated in terms of euclidean spaces
5278 instead of finite cartesian products.
5281 real ^ 'n ~> 'a::real_vector
5282 ~> 'a::euclidean_space
5283 ~> 'a::ordered_euclidean_space
5284 (depends on your needs)
5288 \<chi> x. _ ~> \<chi>\<chi> x. _
5291 Also note that the indices are now natural numbers and not from some
5292 finite type. Finite cartesian products of euclidean spaces, products
5293 of euclidean spaces the real and complex numbers are instantiated to
5294 be euclidean_spaces. INCOMPATIBILITY.
5296 * Session Probability: introduced pextreal as positive extended real
5297 numbers. Use pextreal as value for measures. Introduce the
5298 Radon-Nikodym derivative, product spaces and Fubini's theorem for
5299 arbitrary sigma finite measures. Introduces Lebesgue measure based on
5300 the integral in Multivariate Analysis. INCOMPATIBILITY.
5302 * Session Imperative_HOL: revamped, corrected dozens of inadequacies.
5305 * Session SPARK (with image HOL-SPARK) provides commands to load and
5306 prove verification conditions generated by the SPARK Ada program
5307 verifier. See also src/HOL/SPARK and src/HOL/SPARK/Examples.
5312 * Theorems for additive ring operations (locale abelian_monoid and
5313 descendants) are generated by interpretation from their multiplicative
5314 counterparts. Names (in particular theorem names) have the mandatory
5315 qualifier 'add'. Previous theorem names are redeclared for
5318 * Structure "int_ring" is now an abbreviation (previously a
5319 definition). This fits more natural with advanced interpretations.
5324 * The domain package now runs in definitional mode by default: The
5325 former command 'new_domain' is now called 'domain'. To use the domain
5326 package in its original axiomatic mode, use 'domain (unsafe)'.
5329 * The new class "domain" is now the default sort. Class "predomain"
5330 is an unpointed version of "domain". Theories can be updated by
5331 replacing sort annotations as shown below. INCOMPATIBILITY.
5333 'a::type ~> 'a::countable
5334 'a::cpo ~> 'a::predomain
5335 'a::pcpo ~> 'a::domain
5337 * The old type class "rep" has been superseded by class "domain".
5338 Accordingly, users of the definitional package must remove any
5339 "default_sort rep" declarations. INCOMPATIBILITY.
5341 * The domain package (definitional mode) now supports unpointed
5342 predomain argument types, as long as they are marked 'lazy'. (Strict
5343 arguments must be in class "domain".) For example, the following
5344 domain definition now works:
5346 domain natlist = nil | cons (lazy "nat discr") (lazy "natlist")
5348 * Theory HOLCF/Library/HOL_Cpo provides cpo and predomain class
5349 instances for types from main HOL: bool, nat, int, char, 'a + 'b,
5350 'a option, and 'a list. Additionally, it configures fixrec and the
5351 domain package to work with these types. For example:
5353 fixrec isInl :: "('a + 'b) u -> tr"
5354 where "isInl$(up$(Inl x)) = TT" | "isInl$(up$(Inr y)) = FF"
5356 domain V = VFun (lazy "V -> V") | VCon (lazy "nat") (lazy "V list")
5358 * The "(permissive)" option of fixrec has been replaced with a
5359 per-equation "(unchecked)" option. See
5360 src/HOL/HOLCF/Tutorial/Fixrec_ex.thy for examples. INCOMPATIBILITY.
5362 * The "bifinite" class no longer fixes a constant "approx"; the class
5363 now just asserts that such a function exists. INCOMPATIBILITY.
5365 * Former type "alg_defl" has been renamed to "defl". HOLCF no longer
5366 defines an embedding of type 'a defl into udom by default; instances
5367 of "bifinite" and "domain" classes are available in
5368 src/HOL/HOLCF/Library/Defl_Bifinite.thy.
5370 * The syntax "REP('a)" has been replaced with "DEFL('a)".
5372 * The predicate "directed" has been removed. INCOMPATIBILITY.
5374 * The type class "finite_po" has been removed. INCOMPATIBILITY.
5376 * The function "cprod_map" has been renamed to "prod_map".
5379 * The monadic bind operator on each powerdomain has new binder syntax
5380 similar to sets, e.g. "\<Union>\<sharp>x\<in>xs. t" represents
5381 "upper_bind\<cdot>xs\<cdot>(\<Lambda> x. t)".
5383 * The infix syntax for binary union on each powerdomain has changed
5384 from e.g. "+\<sharp>" to "\<union>\<sharp>", for consistency with set
5385 syntax. INCOMPATIBILITY.
5387 * The constant "UU" has been renamed to "bottom". The syntax "UU" is
5388 still supported as an input translation.
5390 * Renamed some theorems (the original names are also still available).
5392 expand_fun_below ~> fun_below_iff
5393 below_fun_ext ~> fun_belowI
5394 expand_cfun_eq ~> cfun_eq_iff
5395 ext_cfun ~> cfun_eqI
5396 expand_cfun_below ~> cfun_below_iff
5397 below_cfun_ext ~> cfun_belowI
5398 cont2cont_Rep_CFun ~> cont2cont_APP
5400 * The Abs and Rep functions for various types have changed names.
5401 Related theorem names have also changed to match. INCOMPATIBILITY.
5403 Rep_CFun ~> Rep_cfun
5404 Abs_CFun ~> Abs_cfun
5405 Rep_Sprod ~> Rep_sprod
5406 Abs_Sprod ~> Abs_sprod
5407 Rep_Ssum ~> Rep_ssum
5408 Abs_Ssum ~> Abs_ssum
5410 * Lemmas with names of the form *_defined_iff or *_strict_iff have
5411 been renamed to *_bottom_iff. INCOMPATIBILITY.
5413 * Various changes to bisimulation/coinduction with domain package:
5415 - Definitions of "bisim" constants no longer mention definedness.
5416 - With mutual recursion, "bisim" predicate is now curried.
5417 - With mutual recursion, each type gets a separate coind theorem.
5418 - Variable names in bisim_def and coinduct rules have changed.
5422 * Case combinators generated by the domain package for type "foo" are
5423 now named "foo_case" instead of "foo_when". INCOMPATIBILITY.
5425 * Several theorems have been renamed to more accurately reflect the
5426 names of constants and types involved. INCOMPATIBILITY.
5428 thelub_const ~> lub_const
5429 lub_const ~> is_lub_const
5431 is_lub_lub ~> is_lubD2
5433 unique_lub ~> is_lub_unique
5434 is_ub_lub ~> is_lub_rangeD1
5435 lub_bin_chain ~> is_lub_bin_chain
5436 lub_fun ~> is_lub_fun
5437 thelub_fun ~> lub_fun
5438 thelub_cfun ~> lub_cfun
5439 thelub_Pair ~> lub_Pair
5440 lub_cprod ~> is_lub_prod
5441 thelub_cprod ~> lub_prod
5442 minimal_cprod ~> minimal_prod
5443 inst_cprod_pcpo ~> inst_prod_pcpo
5445 compact_UU ~> compact_bottom
5446 deflation_UU ~> deflation_bottom
5447 finite_deflation_UU ~> finite_deflation_bottom
5449 * Many legacy theorem names have been discontinued. INCOMPATIBILITY.
5451 sq_ord_less_eq_trans ~> below_eq_trans
5452 sq_ord_eq_less_trans ~> eq_below_trans
5453 refl_less ~> below_refl
5454 trans_less ~> below_trans
5455 antisym_less ~> below_antisym
5456 antisym_less_inverse ~> po_eq_conv [THEN iffD1]
5457 box_less ~> box_below
5458 rev_trans_less ~> rev_below_trans
5459 not_less2not_eq ~> not_below2not_eq
5460 less_UU_iff ~> below_UU_iff
5461 flat_less_iff ~> flat_below_iff
5462 adm_less ~> adm_below
5463 adm_not_less ~> adm_not_below
5464 adm_compact_not_less ~> adm_compact_not_below
5465 less_fun_def ~> below_fun_def
5466 expand_fun_less ~> fun_below_iff
5467 less_fun_ext ~> fun_belowI
5468 less_discr_def ~> below_discr_def
5469 discr_less_eq ~> discr_below_eq
5470 less_unit_def ~> below_unit_def
5471 less_cprod_def ~> below_prod_def
5472 prod_lessI ~> prod_belowI
5473 Pair_less_iff ~> Pair_below_iff
5474 fst_less_iff ~> fst_below_iff
5475 snd_less_iff ~> snd_below_iff
5476 expand_cfun_less ~> cfun_below_iff
5477 less_cfun_ext ~> cfun_belowI
5478 injection_less ~> injection_below
5479 less_up_def ~> below_up_def
5480 not_Iup_less ~> not_Iup_below
5481 Iup_less ~> Iup_below
5483 Def_inject_less_eq ~> Def_below_Def
5484 Def_less_is_eq ~> Def_below_iff
5485 spair_less_iff ~> spair_below_iff
5486 less_sprod ~> below_sprod
5487 spair_less ~> spair_below
5488 sfst_less_iff ~> sfst_below_iff
5489 ssnd_less_iff ~> ssnd_below_iff
5490 fix_least_less ~> fix_least_below
5491 dist_less_one ~> dist_below_one
5492 less_ONE ~> below_ONE
5493 ONE_less_iff ~> ONE_below_iff
5494 less_sinlD ~> below_sinlD
5495 less_sinrD ~> below_sinrD
5500 * All constant names are now qualified internally and use proper
5501 identifiers, e.g. "IFOL.eq" instead of "op =". INCOMPATIBILITY.
5506 * Antiquotation @{assert} inlines a function bool -> unit that raises
5507 Fail if the argument is false. Due to inlining the source position of
5508 failed assertions is included in the error output.
5510 * Discontinued antiquotation @{theory_ref}, which is obsolete since ML
5511 text is in practice always evaluated with a stable theory checkpoint.
5512 Minor INCOMPATIBILITY, use (Theory.check_thy @{theory}) instead.
5514 * Antiquotation @{theory A} refers to theory A from the ancestry of
5515 the current context, not any accidental theory loader state as before.
5516 Potential INCOMPATIBILITY, subtle change in semantics.
5518 * Syntax.pretty_priority (default 0) configures the required priority
5519 of pretty-printed output and thus affects insertion of parentheses.
5521 * Syntax.default_root (default "any") configures the inner syntax
5522 category (nonterminal symbol) for parsing of terms.
5524 * Former exception Library.UnequalLengths now coincides with
5525 ListPair.UnequalLengths.
5527 * Renamed structure MetaSimplifier to Raw_Simplifier. Note that the
5528 main functionality is provided by structure Simplifier.
5530 * Renamed raw "explode" function to "raw_explode" to emphasize its
5531 meaning. Note that internally to Isabelle, Symbol.explode is used in
5532 almost all situations.
5534 * Discontinued obsolete function sys_error and exception SYS_ERROR.
5535 See implementation manual for further details on exceptions in
5538 * Renamed setmp_noncritical to Unsynchronized.setmp to emphasize its
5541 * Renamed structure PureThy to Pure_Thy and moved most of its
5542 operations to structure Global_Theory, to emphasize that this is
5543 rarely-used global-only stuff.
5545 * Discontinued Output.debug. Minor INCOMPATIBILITY, use plain writeln
5546 instead (or tracing for high-volume output).
5548 * Configuration option show_question_marks only affects regular pretty
5549 printing of types and terms, not raw Term.string_of_vname.
5551 * ML_Context.thm and ML_Context.thms are no longer pervasive. Rare
5552 INCOMPATIBILITY, superseded by static antiquotations @{thm} and
5553 @{thms} for most purposes.
5555 * ML structure Unsynchronized is never opened, not even in Isar
5556 interaction mode as before. Old Unsynchronized.set etc. have been
5557 discontinued -- use plain := instead. This should be *rare* anyway,
5558 since modern tools always work via official context data, notably
5559 configuration options.
5561 * Parallel and asynchronous execution requires special care concerning
5562 interrupts. Structure Exn provides some convenience functions that
5563 avoid working directly with raw Interrupt. User code must not absorb
5564 interrupts -- intermediate handling (for cleanup etc.) needs to be
5565 followed by re-raising of the original exception. Another common
5566 source of mistakes are "handle _" patterns, which make the meaning of
5567 the program subject to physical effects of the environment.
5571 New in Isabelle2009-2 (June 2010)
5572 ---------------------------------
5576 * Authentic syntax for *all* logical entities (type classes, type
5577 constructors, term constants): provides simple and robust
5578 correspondence between formal entities and concrete syntax. Within
5579 the parse tree / AST representations, "constants" are decorated by
5580 their category (class, type, const) and spelled out explicitly with
5581 their full internal name.
5583 Substantial INCOMPATIBILITY concerning low-level syntax declarations
5584 and translations (translation rules and translation functions in ML).
5585 Some hints on upgrading:
5587 - Many existing uses of 'syntax' and 'translations' can be replaced
5588 by more modern 'type_notation', 'notation' and 'abbreviation',
5589 which are independent of this issue.
5591 - 'translations' require markup within the AST; the term syntax
5592 provides the following special forms:
5594 CONST c -- produces syntax version of constant c from context
5595 XCONST c -- literally c, checked as constant from context
5596 c -- literally c, if declared by 'syntax'
5598 Plain identifiers are treated as AST variables -- occasionally the
5599 system indicates accidental variables via the error "rhs contains
5602 Type classes and type constructors are marked according to their
5603 concrete syntax. Some old translations rules need to be written
5604 for the "type" category, using type constructor application
5605 instead of pseudo-term application of the default category
5608 - 'parse_translation' etc. in ML may use the following
5611 @{class_syntax c} -- type class c within parse tree / AST
5612 @{term_syntax c} -- type constructor c within parse tree / AST
5613 @{const_syntax c} -- ML version of "CONST c" above
5614 @{syntax_const c} -- literally c (checked wrt. 'syntax' declarations)
5616 - Literal types within 'typed_print_translations', i.e. those *not*
5617 represented as pseudo-terms are represented verbatim. Use @{class
5618 c} or @{type_name c} here instead of the above syntax
5621 Note that old non-authentic syntax was based on unqualified base
5622 names, so all of the above "constant" names would coincide. Recall
5623 that 'print_syntax' and ML_command "set Syntax.trace_ast" help to
5624 diagnose syntax problems.
5626 * Type constructors admit general mixfix syntax, not just infix.
5628 * Concrete syntax may be attached to local entities without a proof
5629 body, too. This works via regular mixfix annotations for 'fix',
5630 'def', 'obtain' etc. or via the explicit 'write' command, which is
5631 similar to the 'notation' command in theory specifications.
5633 * Discontinued unnamed infix syntax (legacy feature for many years) --
5634 need to specify constant name and syntax separately. Internal ML
5635 datatype constructors have been renamed from InfixName to Infix etc.
5636 Minor INCOMPATIBILITY.
5638 * Schematic theorem statements need to be explicitly markup as such,
5639 via commands 'schematic_lemma', 'schematic_theorem',
5640 'schematic_corollary'. Thus the relevance of the proof is made
5641 syntactically clear, which impacts performance in a parallel or
5642 asynchronous interactive environment. Minor INCOMPATIBILITY.
5644 * Use of cumulative prems via "!" in some proof methods has been
5645 discontinued (old legacy feature).
5647 * References 'trace_simp' and 'debug_simp' have been replaced by
5648 configuration options stored in the context. Enabling tracing (the
5649 case of debugging is similar) in proofs works via
5651 using [[trace_simp = true]]
5653 Tracing is then active for all invocations of the simplifier in
5654 subsequent goal refinement steps. Tracing may also still be enabled or
5655 disabled via the ProofGeneral settings menu.
5657 * Separate commands 'hide_class', 'hide_type', 'hide_const',
5658 'hide_fact' replace the former 'hide' KIND command. Minor
5661 * Improved parallelism of proof term normalization: usedir -p2 -q0 is
5662 more efficient than combinations with -q1 or -q2.
5667 * Proofterms record type-class reasoning explicitly, using the
5668 "unconstrain" operation internally. This eliminates all sort
5669 constraints from a theorem and proof, introducing explicit
5670 OFCLASS-premises. On the proof term level, this operation is
5671 automatically applied at theorem boundaries, such that closed proofs
5672 are always free of sort constraints. INCOMPATIBILITY for tools that
5673 inspect proof terms.
5675 * Local theory specifications may depend on extra type variables that
5676 are not present in the result type -- arguments TYPE('a) :: 'a itself
5677 are added internally. For example:
5679 definition unitary :: bool where "unitary = (ALL (x::'a) y. x = y)"
5681 * Predicates of locales introduced by classes carry a mandatory
5682 "class" prefix. INCOMPATIBILITY.
5684 * Vacuous class specifications observe default sort. INCOMPATIBILITY.
5686 * Old 'axclass' command has been discontinued. INCOMPATIBILITY, use
5689 * Command 'code_reflect' allows to incorporate generated ML code into
5690 runtime environment; replaces immature code_datatype antiquotation.
5693 * Code generator: simple concept for abstract datatypes obeying
5696 * Code generator: details of internal data cache have no impact on the
5697 user space functionality any longer.
5699 * Methods "unfold_locales" and "intro_locales" ignore non-locale
5700 subgoals. This is more appropriate for interpretations with 'where'.
5703 * Command 'example_proof' opens an empty proof body. This allows to
5704 experiment with Isar, without producing any persistent result.
5706 * Commands 'type_notation' and 'no_type_notation' declare type syntax
5707 within a local theory context, with explicit checking of the
5708 constructors involved (in contrast to the raw 'syntax' versions).
5710 * Commands 'types' and 'typedecl' now work within a local theory
5711 context -- without introducing dependencies on parameters or
5712 assumptions, which is not possible in Isabelle/Pure.
5714 * Command 'defaultsort' has been renamed to 'default_sort', it works
5715 within a local theory context. Minor INCOMPATIBILITY.
5720 * Command 'typedef' now works within a local theory context -- without
5721 introducing dependencies on parameters or assumptions, which is not
5722 possible in Isabelle/Pure/HOL. Note that the logical environment may
5723 contain multiple interpretations of local typedefs (with different
5724 non-emptiness proofs), even in a global theory context.
5726 * New package for quotient types. Commands 'quotient_type' and
5727 'quotient_definition' may be used for defining types and constants by
5728 quotient constructions. An example is the type of integers created by
5729 quotienting pairs of natural numbers:
5732 intrel :: "(nat * nat) => (nat * nat) => bool"
5734 "intrel (x, y) (u, v) = (x + v = u + y)"
5736 quotient_type int = "nat * nat" / intrel
5737 by (auto simp add: equivp_def expand_fun_eq)
5740 "0::int" is "(0::nat, 0::nat)"
5742 The method "lifting" can be used to lift of theorems from the
5743 underlying "raw" type to the quotient type. The example
5744 src/HOL/Quotient_Examples/FSet.thy includes such a quotient
5745 construction and provides a reasoning infrastructure for finite sets.
5747 * Renamed Library/Quotient.thy to Library/Quotient_Type.thy to avoid
5748 clash with new theory Quotient in Main HOL.
5750 * Moved the SMT binding into the main HOL session, eliminating
5751 separate HOL-SMT session.
5753 * List membership infix mem operation is only an input abbreviation.
5756 * Theory Library/Word.thy has been removed. Use library Word/Word.thy
5757 for future developements; former Library/Word.thy is still present in
5758 the AFP entry RSAPPS.
5760 * Theorem Int.int_induct renamed to Int.int_of_nat_induct and is no
5761 longer shadowed. INCOMPATIBILITY.
5763 * Dropped theorem duplicate comp_arith; use semiring_norm instead.
5766 * Dropped theorem RealPow.real_sq_order; use power2_le_imp_le instead.
5769 * Dropped normalizing_semiring etc; use the facts in semiring classes
5770 instead. INCOMPATIBILITY.
5772 * Dropped several real-specific versions of lemmas about floor and
5773 ceiling; use the generic lemmas from theory "Archimedean_Field"
5774 instead. INCOMPATIBILITY.
5776 floor_number_of_eq ~> floor_number_of
5777 le_floor_eq_number_of ~> number_of_le_floor
5778 le_floor_eq_zero ~> zero_le_floor
5779 le_floor_eq_one ~> one_le_floor
5780 floor_less_eq_number_of ~> floor_less_number_of
5781 floor_less_eq_zero ~> floor_less_zero
5782 floor_less_eq_one ~> floor_less_one
5783 less_floor_eq_number_of ~> number_of_less_floor
5784 less_floor_eq_zero ~> zero_less_floor
5785 less_floor_eq_one ~> one_less_floor
5786 floor_le_eq_number_of ~> floor_le_number_of
5787 floor_le_eq_zero ~> floor_le_zero
5788 floor_le_eq_one ~> floor_le_one
5789 floor_subtract_number_of ~> floor_diff_number_of
5790 floor_subtract_one ~> floor_diff_one
5791 ceiling_number_of_eq ~> ceiling_number_of
5792 ceiling_le_eq_number_of ~> ceiling_le_number_of
5793 ceiling_le_zero_eq ~> ceiling_le_zero
5794 ceiling_le_eq_one ~> ceiling_le_one
5795 less_ceiling_eq_number_of ~> number_of_less_ceiling
5796 less_ceiling_eq_zero ~> zero_less_ceiling
5797 less_ceiling_eq_one ~> one_less_ceiling
5798 ceiling_less_eq_number_of ~> ceiling_less_number_of
5799 ceiling_less_eq_zero ~> ceiling_less_zero
5800 ceiling_less_eq_one ~> ceiling_less_one
5801 le_ceiling_eq_number_of ~> number_of_le_ceiling
5802 le_ceiling_eq_zero ~> zero_le_ceiling
5803 le_ceiling_eq_one ~> one_le_ceiling
5804 ceiling_subtract_number_of ~> ceiling_diff_number_of
5805 ceiling_subtract_one ~> ceiling_diff_one
5807 * Theory "Finite_Set": various folding_XXX locales facilitate the
5808 application of the various fold combinators on finite sets.
5810 * Library theory "RBT" renamed to "RBT_Impl"; new library theory "RBT"
5811 provides abstract red-black tree type which is backed by "RBT_Impl" as
5812 implementation. INCOMPATIBILITY.
5814 * Theory Library/Coinductive_List has been removed -- superseded by
5815 AFP/thys/Coinductive.
5817 * Theory PReal, including the type "preal" and related operations, has
5818 been removed. INCOMPATIBILITY.
5820 * Real: new development using Cauchy Sequences.
5822 * Split off theory "Big_Operators" containing setsum, setprod,
5823 Inf_fin, Sup_fin, Min, Max from theory Finite_Set. INCOMPATIBILITY.
5825 * Theory "Rational" renamed to "Rat", for consistency with "Nat",
5826 "Int" etc. INCOMPATIBILITY.
5828 * Constant Rat.normalize needs to be qualified. INCOMPATIBILITY.
5830 * New set of rules "ac_simps" provides combined assoc / commute
5831 rewrites for all interpretations of the appropriate generic locales.
5833 * Renamed theory "OrderedGroup" to "Groups" and split theory
5834 "Ring_and_Field" into theories "Rings" and "Fields"; for more
5835 appropriate and more consistent names suitable for name prefixes
5836 within the HOL theories. INCOMPATIBILITY.
5838 * Some generic constants have been put to appropriate theories:
5839 - less_eq, less: Orderings
5840 - zero, one, plus, minus, uminus, times, abs, sgn: Groups
5841 - inverse, divide: Rings
5844 * More consistent naming of type classes involving orderings (and
5847 lower_semilattice ~> semilattice_inf
5848 upper_semilattice ~> semilattice_sup
5850 dense_linear_order ~> dense_linorder
5852 pordered_ab_group_add ~> ordered_ab_group_add
5853 pordered_ab_group_add_abs ~> ordered_ab_group_add_abs
5854 pordered_ab_semigroup_add ~> ordered_ab_semigroup_add
5855 pordered_ab_semigroup_add_imp_le ~> ordered_ab_semigroup_add_imp_le
5856 pordered_cancel_ab_semigroup_add ~> ordered_cancel_ab_semigroup_add
5857 pordered_cancel_comm_semiring ~> ordered_cancel_comm_semiring
5858 pordered_cancel_semiring ~> ordered_cancel_semiring
5859 pordered_comm_monoid_add ~> ordered_comm_monoid_add
5860 pordered_comm_ring ~> ordered_comm_ring
5861 pordered_comm_semiring ~> ordered_comm_semiring
5862 pordered_ring ~> ordered_ring
5863 pordered_ring_abs ~> ordered_ring_abs
5864 pordered_semiring ~> ordered_semiring
5866 ordered_ab_group_add ~> linordered_ab_group_add
5867 ordered_ab_semigroup_add ~> linordered_ab_semigroup_add
5868 ordered_cancel_ab_semigroup_add ~> linordered_cancel_ab_semigroup_add
5869 ordered_comm_semiring_strict ~> linordered_comm_semiring_strict
5870 ordered_field ~> linordered_field
5871 ordered_field_no_lb ~> linordered_field_no_lb
5872 ordered_field_no_ub ~> linordered_field_no_ub
5873 ordered_field_dense_linear_order ~> dense_linordered_field
5874 ordered_idom ~> linordered_idom
5875 ordered_ring ~> linordered_ring
5876 ordered_ring_le_cancel_factor ~> linordered_ring_le_cancel_factor
5877 ordered_ring_less_cancel_factor ~> linordered_ring_less_cancel_factor
5878 ordered_ring_strict ~> linordered_ring_strict
5879 ordered_semidom ~> linordered_semidom
5880 ordered_semiring ~> linordered_semiring
5881 ordered_semiring_1 ~> linordered_semiring_1
5882 ordered_semiring_1_strict ~> linordered_semiring_1_strict
5883 ordered_semiring_strict ~> linordered_semiring_strict
5885 The following slightly odd type classes have been moved to a
5886 separate theory Library/Lattice_Algebras:
5888 lordered_ab_group_add ~> lattice_ab_group_add
5889 lordered_ab_group_add_abs ~> lattice_ab_group_add_abs
5890 lordered_ab_group_add_meet ~> semilattice_inf_ab_group_add
5891 lordered_ab_group_add_join ~> semilattice_sup_ab_group_add
5892 lordered_ring ~> lattice_ring
5896 * Refined field classes:
5897 - classes division_ring_inverse_zero, field_inverse_zero,
5898 linordered_field_inverse_zero include rule inverse 0 = 0 --
5899 subsumes former division_by_zero class;
5900 - numerous lemmas have been ported from field to division_ring.
5903 * Refined algebra theorem collections:
5904 - dropped theorem group group_simps, use algebra_simps instead;
5905 - dropped theorem group ring_simps, use field_simps instead;
5906 - proper theorem collection field_simps subsumes former theorem
5907 groups field_eq_simps and field_simps;
5908 - dropped lemma eq_minus_self_iff which is a duplicate for
5912 * Theory Finite_Set and List: some lemmas have been generalized from
5915 fun_left_comm_idem_inter ~> fun_left_comm_idem_inf
5916 fun_left_comm_idem_union ~> fun_left_comm_idem_sup
5917 inter_Inter_fold_inter ~> inf_Inf_fold_inf
5918 union_Union_fold_union ~> sup_Sup_fold_sup
5919 Inter_fold_inter ~> Inf_fold_inf
5920 Union_fold_union ~> Sup_fold_sup
5921 inter_INTER_fold_inter ~> inf_INFI_fold_inf
5922 union_UNION_fold_union ~> sup_SUPR_fold_sup
5923 INTER_fold_inter ~> INFI_fold_inf
5924 UNION_fold_union ~> SUPR_fold_sup
5926 * Theory "Complete_Lattice": lemmas top_def and bot_def have been
5927 replaced by the more convenient lemmas Inf_empty and Sup_empty.
5928 Dropped lemmas Inf_insert_simp and Sup_insert_simp, which are subsumed
5929 by Inf_insert and Sup_insert. Lemmas Inf_UNIV and Sup_UNIV replace
5930 former Inf_Univ and Sup_Univ. Lemmas inf_top_right and sup_bot_right
5931 subsume inf_top and sup_bot respectively. INCOMPATIBILITY.
5933 * Reorganized theory Multiset: swapped notation of pointwise and
5936 - pointwise ordering is instance of class order with standard syntax
5938 - multiset ordering has syntax <=# and <#; partial order properties
5939 are provided by means of interpretation with prefix
5941 - less duplication, less historical organization of sections,
5942 conversion from associations lists to multisets, rudimentary code
5944 - use insert_DiffM2 [symmetric] instead of elem_imp_eq_diff_union,
5949 multiset_eq_conv_count_eq ~> multiset_ext_iff
5950 multi_count_ext ~> multiset_ext
5951 diff_union_inverse2 ~> diff_union_cancelR
5955 * Theory Permutation: replaced local "remove" by List.remove1.
5957 * Code generation: ML and OCaml code is decorated with signatures.
5959 * Theory List: added transpose.
5961 * Library/Nat_Bijection.thy is a collection of bijective functions
5962 between nat and other types, which supersedes the older libraries
5963 Library/Nat_Int_Bij.thy and HOLCF/NatIso.thy. INCOMPATIBILITY.
5966 Nat_Int_Bij.nat2_to_nat ~> prod_encode
5967 Nat_Int_Bij.nat_to_nat2 ~> prod_decode
5968 Nat_Int_Bij.int_to_nat_bij ~> int_encode
5969 Nat_Int_Bij.nat_to_int_bij ~> int_decode
5970 Countable.pair_encode ~> prod_encode
5971 NatIso.prod2nat ~> prod_encode
5972 NatIso.nat2prod ~> prod_decode
5973 NatIso.sum2nat ~> sum_encode
5974 NatIso.nat2sum ~> sum_decode
5975 NatIso.list2nat ~> list_encode
5976 NatIso.nat2list ~> list_decode
5977 NatIso.set2nat ~> set_encode
5978 NatIso.nat2set ~> set_decode
5981 Nat_Int_Bij.bij_nat_to_int_bij ~> bij_int_decode
5982 Nat_Int_Bij.nat2_to_nat_inj ~> inj_prod_encode
5983 Nat_Int_Bij.nat2_to_nat_surj ~> surj_prod_encode
5984 Nat_Int_Bij.nat_to_nat2_inj ~> inj_prod_decode
5985 Nat_Int_Bij.nat_to_nat2_surj ~> surj_prod_decode
5986 Nat_Int_Bij.i2n_n2i_id ~> int_encode_inverse
5987 Nat_Int_Bij.n2i_i2n_id ~> int_decode_inverse
5988 Nat_Int_Bij.surj_nat_to_int_bij ~> surj_int_encode
5989 Nat_Int_Bij.surj_int_to_nat_bij ~> surj_int_decode
5990 Nat_Int_Bij.inj_nat_to_int_bij ~> inj_int_encode
5991 Nat_Int_Bij.inj_int_to_nat_bij ~> inj_int_decode
5992 Nat_Int_Bij.bij_nat_to_int_bij ~> bij_int_encode
5993 Nat_Int_Bij.bij_int_to_nat_bij ~> bij_int_decode
5996 - Renamed ATP commands:
5997 atp_info ~> sledgehammer running_atps
5998 atp_kill ~> sledgehammer kill_atps
5999 atp_messages ~> sledgehammer messages
6000 atp_minimize ~> sledgehammer minimize
6001 print_atps ~> sledgehammer available_atps
6003 - Added user's manual ("isabelle doc sledgehammer").
6004 - Added option syntax and "sledgehammer_params" to customize
6005 Sledgehammer's behavior. See the manual for details.
6006 - Modified the Isar proof reconstruction code so that it produces
6007 direct proofs rather than proofs by contradiction. (This feature
6008 is still experimental.)
6009 - Made Isar proof reconstruction work for SPASS, remote ATPs, and in
6011 - Added support for TPTP syntax for SPASS via the "spass_tptp" ATP.
6014 - Added and implemented "binary_ints" and "bits" options.
6015 - Added "std" option and implemented support for nonstandard models.
6016 - Added and implemented "finitize" option to improve the precision
6017 of infinite datatypes based on a monotonicity analysis.
6018 - Added support for quotient types.
6019 - Added support for "specification" and "ax_specification"
6021 - Added support for local definitions (for "function" and
6022 "termination" proofs).
6023 - Added support for term postprocessors.
6024 - Optimized "Multiset.multiset" and "FinFun.finfun".
6025 - Improved efficiency of "destroy_constrs" optimization.
6026 - Fixed soundness bugs related to "destroy_constrs" optimization and
6028 - Fixed soundness bug related to higher-order constructors.
6029 - Fixed soundness bug when "full_descrs" is enabled.
6030 - Improved precision of set constructs.
6031 - Added "atoms" option.
6032 - Added cache to speed up repeated Kodkod invocations on the same
6034 - Renamed "MiniSatJNI", "zChaffJNI", "BerkMinAlloy", and
6035 "SAT4JLight" to "MiniSat_JNI", "zChaff_JNI", "BerkMin_Alloy", and
6036 "SAT4J_Light". INCOMPATIBILITY.
6037 - Removed "skolemize", "uncurry", "sym_break", "flatten_prop",
6038 "sharing_depth", and "show_skolems" options. INCOMPATIBILITY.
6039 - Removed "nitpick_intro" attribute. INCOMPATIBILITY.
6041 * Method "induct" now takes instantiations of the form t, where t is not
6042 a variable, as a shorthand for "x == t", where x is a fresh variable.
6043 If this is not intended, t has to be enclosed in parentheses.
6044 By default, the equalities generated by definitional instantiations
6045 are pre-simplified, which may cause parameters of inductive cases
6046 to disappear, or may even delete some of the inductive cases.
6047 Use "induct (no_simp)" instead of "induct" to restore the old
6048 behaviour. The (no_simp) option is also understood by the "cases"
6049 and "nominal_induct" methods, which now perform pre-simplification, too.
6055 * Variable names in lemmas generated by the domain package have
6056 changed; the naming scheme is now consistent with the HOL datatype
6057 package. Some proof scripts may be affected, INCOMPATIBILITY.
6059 * The domain package no longer defines the function "foo_copy" for
6060 recursive domain "foo". The reach lemma is now stated directly in
6061 terms of "foo_take". Lemmas and proofs that mention "foo_copy" must
6062 be reformulated in terms of "foo_take", INCOMPATIBILITY.
6064 * Most definedness lemmas generated by the domain package (previously
6065 of the form "x ~= UU ==> foo$x ~= UU") now have an if-and-only-if form
6066 like "foo$x = UU <-> x = UU", which works better as a simp rule.
6067 Proofs that used definedness lemmas as intro rules may break,
6068 potential INCOMPATIBILITY.
6070 * Induction and casedist rules generated by the domain package now
6071 declare proper case_names (one called "bottom", and one named for each
6072 constructor). INCOMPATIBILITY.
6074 * For mutually-recursive domains, separate "reach" and "take_lemma"
6075 rules are generated for each domain, INCOMPATIBILITY.
6077 foo_bar.reach ~> foo.reach bar.reach
6078 foo_bar.take_lemmas ~> foo.take_lemma bar.take_lemma
6080 * Some lemmas generated by the domain package have been renamed for
6081 consistency with the datatype package, INCOMPATIBILITY.
6083 foo.ind ~> foo.induct
6084 foo.finite_ind ~> foo.finite_induct
6085 foo.coind ~> foo.coinduct
6086 foo.casedist ~> foo.exhaust
6087 foo.exhaust ~> foo.nchotomy
6089 * For consistency with other definition packages, the fixrec package
6090 now generates qualified theorem names, INCOMPATIBILITY.
6092 foo_simps ~> foo.simps
6093 foo_unfold ~> foo.unfold
6094 foo_induct ~> foo.induct
6096 * The "fixrec_simp" attribute has been removed. The "fixrec_simp"
6097 method and internal fixrec proofs now use the default simpset instead.
6100 * The "contlub" predicate has been removed. Proof scripts should use
6101 lemma contI2 in place of monocontlub2cont, INCOMPATIBILITY.
6103 * The "admw" predicate has been removed, INCOMPATIBILITY.
6105 * The constants cpair, cfst, and csnd have been removed in favor of
6106 Pair, fst, and snd from Isabelle/HOL, INCOMPATIBILITY.
6111 * Antiquotations for basic formal entities:
6113 @{class NAME} -- type class
6114 @{class_syntax NAME} -- syntax representation of the above
6116 @{type_name NAME} -- logical type
6117 @{type_abbrev NAME} -- type abbreviation
6118 @{nonterminal NAME} -- type of concrete syntactic category
6119 @{type_syntax NAME} -- syntax representation of any of the above
6121 @{const_name NAME} -- logical constant (INCOMPATIBILITY)
6122 @{const_abbrev NAME} -- abbreviated constant
6123 @{const_syntax NAME} -- syntax representation of any of the above
6125 * Antiquotation @{syntax_const NAME} ensures that NAME refers to a raw
6126 syntax constant (cf. 'syntax' command).
6128 * Antiquotation @{make_string} inlines a function to print arbitrary
6129 values similar to the ML toplevel. The result is compiler dependent
6130 and may fall back on "?" in certain situations.
6132 * Diagnostic commands 'ML_val' and 'ML_command' may refer to
6133 antiquotations @{Isar.state} and @{Isar.goal}. This replaces impure
6134 Isar.state() and Isar.goal(), which belong to the old TTY loop and do
6135 not work with the asynchronous Isar document model.
6137 * Configuration options now admit dynamic default values, depending on
6138 the context or even global references.
6140 * SHA1.digest digests strings according to SHA-1 (see RFC 3174). It
6141 uses an efficient external library if available (for Poly/ML).
6143 * Renamed some important ML structures, while keeping the old names
6144 for some time as aliases within the structure Legacy:
6146 OuterKeyword ~> Keyword
6149 OuterSyntax ~> Outer_Syntax
6150 PrintMode ~> Print_Mode
6151 SpecParse ~> Parse_Spec
6154 ThyOutput ~> Thy_Output
6155 TypeInfer ~> Type_Infer
6157 Note that "open Legacy" simplifies porting of sources, but forgetting
6158 to remove it again will complicate porting again in the future.
6160 * Most operations that refer to a global context are named
6161 accordingly, e.g. Simplifier.global_context or
6162 ProofContext.init_global. There are some situations where a global
6163 context actually works, but under normal circumstances one needs to
6164 pass the proper local context through the code!
6166 * Discontinued old TheoryDataFun with its copy/init operation -- data
6167 needs to be pure. Functor Theory_Data_PP retains the traditional
6168 Pretty.pp argument to merge, which is absent in the standard
6169 Theory_Data version.
6171 * Sorts.certify_sort and derived "cert" operations for types and terms
6172 no longer minimize sorts. Thus certification at the boundary of the
6173 inference kernel becomes invariant under addition of class relations,
6174 which is an important monotonicity principle. Sorts are now minimized
6175 in the syntax layer only, at the boundary between the end-user and the
6176 system. Subtle INCOMPATIBILITY, may have to use Sign.minimize_sort
6177 explicitly in rare situations.
6179 * Renamed old-style Drule.standard to Drule.export_without_context, to
6180 emphasize that this is in no way a standard operation.
6183 * Subgoal.FOCUS (and variants): resulting goal state is normalized as
6184 usual for resolution. Rare INCOMPATIBILITY.
6186 * Renamed varify/unvarify operations to varify_global/unvarify_global
6187 to emphasize that these only work in a global situation (which is
6190 * Curried take and drop in library.ML; negative length is interpreted
6191 as infinity (as in chop). Subtle INCOMPATIBILITY.
6193 * Proof terms: type substitutions on proof constants now use canonical
6194 order of type variables. INCOMPATIBILITY for tools working with proof
6197 * Raw axioms/defs may no longer carry sort constraints, and raw defs
6198 may no longer carry premises. User-level specifications are
6199 transformed accordingly by Thm.add_axiom/add_def.
6204 * Discontinued special HOL_USEDIR_OPTIONS for the main HOL image;
6205 ISABELLE_USEDIR_OPTIONS applies uniformly to all sessions. Note that
6206 proof terms are enabled unconditionally in the new HOL-Proofs image.
6208 * Discontinued old ISABELLE and ISATOOL environment settings (legacy
6209 feature since Isabelle2009). Use ISABELLE_PROCESS and ISABELLE_TOOL,
6212 * Old lib/scripts/polyml-platform is superseded by the
6213 ISABELLE_PLATFORM setting variable, which defaults to the 32 bit
6214 variant, even on a 64 bit machine. The following example setting
6215 prefers 64 bit if available:
6217 ML_PLATFORM="${ISABELLE_PLATFORM64:-$ISABELLE_PLATFORM}"
6219 * The preliminary Isabelle/jEdit application demonstrates the emerging
6220 Isabelle/Scala layer for advanced prover interaction and integration.
6221 See src/Tools/jEdit or "isabelle jedit" provided by the properly built
6224 * "IsabelleText" is a Unicode font derived from Bitstream Vera Mono
6225 and Bluesky TeX fonts. It provides the usual Isabelle symbols,
6226 similar to the default assignment of the document preparation system
6227 (cf. isabellesym.sty). The Isabelle/Scala class Isabelle_System
6228 provides some operations for direct access to the font without asking
6229 the user for manual installation.
6233 New in Isabelle2009-1 (December 2009)
6234 -------------------------------------
6238 * Discontinued old form of "escaped symbols" such as \\<forall>. Only
6239 one backslash should be used, even in ML sources.
6244 * Locale interpretation propagates mixins along the locale hierarchy.
6245 The currently only available mixins are the equations used to map
6246 local definitions to terms of the target domain of an interpretation.
6248 * Reactivated diagnostic command 'print_interps'. Use "print_interps
6249 loc" to print all interpretations of locale "loc" in the theory.
6250 Interpretations in proofs are not shown.
6252 * Thoroughly revised locales tutorial. New section on conditional
6255 * On instantiation of classes, remaining undefined class parameters
6256 are formally declared. INCOMPATIBILITY.
6259 *** Document preparation ***
6261 * New generalized style concept for printing terms: @{foo (style) ...}
6262 instead of @{foo_style style ...} (old form is still retained for
6263 backward compatibility). Styles can be also applied for
6264 antiquotations prop, term_type and typeof.
6269 * New proof method "smt" for a combination of first-order logic with
6270 equality, linear and nonlinear (natural/integer/real) arithmetic, and
6271 fixed-size bitvectors; there is also basic support for higher-order
6272 features (esp. lambda abstractions). It is an incomplete decision
6273 procedure based on external SMT solvers using the oracle mechanism;
6274 for the SMT solver Z3, this method is proof-producing. Certificates
6275 are provided to avoid calling the external solvers solely for
6276 re-checking proofs. Due to a remote SMT service there is no need for
6277 installing SMT solvers locally. See src/HOL/SMT.
6279 * New commands to load and prove verification conditions generated by
6280 the Boogie program verifie