doc-src/ERRATA.txt
author lcp
Fri, 11 Nov 1994 10:31:51 +0100
changeset 701 74ee8b9ff9a7
parent 614 da97045ef59a
child 716 79adbdbda0fb
permissions -rw-r--r--
argument swaps in HOL
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     1
$Id$
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     2
ERRATA in the book "Isabelle: A Generic Theorem Prover"
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     3
by Lawrence C. Paulson (contributions by Tobias Nipkow)
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     4
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     5
Some of these errors are typographical but most of them are due to continuing
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
     6
changes to Isabelle.
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
     7
491
1a7717eca145 logics update
lcp
parents: 479
diff changeset
     8
Thanks to Sara Kalvala, Tobias Nipkow
1a7717eca145 logics update
lcp
parents: 479
diff changeset
     9
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    10
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    11
INTRODUCTION TO ISABELLE
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    12
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    13
Advanced Methods
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    14
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    15
page 52, middle: the declaration "types bool,nat" should be "types bool nat"
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    16
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    17
page 57, bottom: should be addsimps in 
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    18
	val add_ss = FOL_ss addrews [add_0, add_Suc]
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    19
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    20
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    21
ISABELLE REFERENCE MANUAL
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    22
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    23
Introduction
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    24
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    25
page 67: show_brackets is another flag, controlling display of bracketting
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    26
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    27
Tactics
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    28
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    29
page 85: subgoals_tac is another tactic, for multiple calls to subgoal_tac
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    30
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    31
Theories
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    32
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    33
page 117: the three lines of ML shown can be abbreviated to just
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    34
	init_thy_reader();
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    35
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    36
page 118: extend_theory has been replaced by numerous functions for adding
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    37
types, constants, axioms, etc.
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    38
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    39
Defining Logics
507
a00301e9e64b addition of show_brackets
lcp
parents: 491
diff changeset
    40
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    41
page 127: type constraints ("::") now have a very low priority of 4.
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    42
As in ML, they must usually be enclosed in paretheses.
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    43
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    44
Syntax Transformations
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    45
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    46
page 145, line -5: delete repeated "the" in "before the the .thy file"
507
a00301e9e64b addition of show_brackets
lcp
parents: 491
diff changeset
    47
a00301e9e64b addition of show_brackets
lcp
parents: 491
diff changeset
    48
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    49
ISABELLE'S OBJECT-LOGICS
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    50
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    51
Zermelo-Fraenkel Set Theory
507
a00301e9e64b addition of show_brackets
lcp
parents: 491
diff changeset
    52
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    53
page 209: axioms have been renamed:
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    54
	union_iff is now Union_iff
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    55
	power_set is now Pow_iff
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    56
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    57
page 215, bottom of figure 17.10: DiffD2 is now  "c : A - B ==> c ~: B"
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    58
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    59
page 215, bottom: rules mem_anti_sym and mem_anti_refl are now mem_asym and
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    60
mem_irrefl
456
f1df7fc211a7 New errata list for the documentation
lcp
parents:
diff changeset
    61
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    62
page 222, top: missing braces in qconverse_def (around right-hand side)
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    63
and QSigma_def (around <x;y>)
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    64
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    65
page 223, top: lfp_def, gfp_def have missing braces around the argument of
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    66
Inter, Union
458
877704b91847 type constraints
nipkow
parents: 456
diff changeset
    67
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    68
page 228: now there is also a theory of cardinal numbers and some
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    69
developments involving the Axiom of Choice.
479
db5a95f2952e *** empty log message ***
nipkow
parents: 458
diff changeset
    70
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    71
page 229: now there is another examples directory, IMP (a semantics
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    72
equivalence proof for an imperative language)
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    73
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    74
Higher-Order Logic
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    75
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    76
page 243: Pow is a new constant of type 'a set => 'a set set
491
1a7717eca145 logics update
lcp
parents: 479
diff changeset
    77
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    78
page 246: Pow is defined by   Pow(A) == {B. B <= A}
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    79
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    80
page 248: Pow has the rules
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    81
	PowI     A<=B ==> A: Pow(B)
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
    82
	PowD     A: Pow(B) ==> A<=B
507
a00301e9e64b addition of show_brackets
lcp
parents: 491
diff changeset
    83
701
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    84
page 251: split now has type [['a,'b] => 'c, 'a * 'b] => 'c
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    85
Definition modified accordingly
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    86
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    87
page 252: sum_case now has type ['a=>'c,'b=>'c, 'a+'b] =>'c
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    88
Definition and rules modified accordingly
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    89
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    90
page 254: nat_case now has type ['a, nat=>'a, nat] =>'a
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    91
Definition modified accordingly
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    92
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    93
page 256,258: list_case now takes the list as its last argument, not the
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    94
first.
74ee8b9ff9a7 argument swaps in HOL
lcp
parents: 614
diff changeset
    95
601
208834a9ba70 Added primrec section
nipkow
parents: 599
diff changeset
    96
page 259: HOL theory files may now include datatype declarations, primitive
614
da97045ef59a now mentions that the sections are available as
lcp
parents: 601
diff changeset
    97
recursive function definitions, and (co)inductive definitions.  (These new
da97045ef59a now mentions that the sections are available as
lcp
parents: 601
diff changeset
    98
sections are available separately as the file ml/HOL-extensions.dvi.gz,
da97045ef59a now mentions that the sections are available as
lcp
parents: 601
diff changeset
    99
host ftp.cl.cam.ac.uk.)
599
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
   100
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
   101
page 259: now there is another examples directory, IMP (a semantics
08b403fe92b1 now in a format that could be published
lcp
parents: 507
diff changeset
   102
equivalence proof for an imperative language)