diff -r 73fb6a200e36 -r 2ac9265b2cd5 NEWS --- a/NEWS Wed Feb 27 15:23:42 2002 +0100 +++ b/NEWS Wed Feb 27 18:41:28 2002 +0100 @@ -87,7 +87,9 @@ version by Florian Kammüller, Isar locales package high-level proof contexts rather than raw logical ones (e.g. we admit to include attributes everywhere); operations on locales include merge and -rename; e.g. see HOL/ex/Locales.thy; +rename; support for implicit arguments (``structures''); simultaneous +type-inference over imports and text; see also HOL/ex/Locales.thy for +some examples; * Pure: the following commands have been ``localized'', supporting a target locale specification "(in name)": 'lemma', 'theorem', @@ -95,12 +97,24 @@ stored both within the locale and at the theory level (exported and qualified by the locale name); -* Pure: theory goals now support ad-hoc contexts, which are discharged -in the result, as in ``lemma (assumes A and B) K: A .''; syntax -coincides with that of a locale body; +* Pure: theory goals may now be specified in ``long'' form, with +ad-hoc contexts consisting of arbitrary locale elements. for example +``lemma foo: fixes x assumes "A x" shows "B x"'' (local syntax and +definitions may be given, too); the result is a meta-level rule with +the context elements being discharged in the obvious way; + +* Pure: new proof command 'using' allows to augment currently used +facts after a goal statement ('using' is syntactically analogous to +'apply', but acts on the goal's facts only); this allows chained facts +to be separated into parts given before and after a claim, as in +``from a and b have C using d and e ''; * Pure: renamed "antecedent" case to "rule_context"; +* Pure: new 'judgment' command records explicit information about the +object-logic embedding (used by several tools internally); no longer +use hard-wired "Trueprop"; + * Pure: added 'corollary' command; * Pure: fixed 'token_translation' command;