# HG changeset patch # User wenzelm # Date 1661024095 -7200 # Node ID 06eb4d0031e32b36419341b1b5fa8ce96b92b7ff # Parent d7e0b6620c07dbaea29b1d9d11f2d6fbba22f69d# Parent 4586e90573acaf96b798dbca4ac6df31dc540e06 merged; diff -r d7e0b6620c07 -r 06eb4d0031e3 NEWS --- a/NEWS Fri Aug 19 05:49:17 2022 +0000 +++ b/NEWS Sat Aug 20 21:34:55 2022 +0200 @@ -202,6 +202,10 @@ *** System *** +* HTML presentation no longer supports README.html, which was meant as +add-on to the index.html of a session. Rare INCOMPATIBILITY, consider +using a separate theory "README" with Isabelle document markup/markdown. + * Isabelle/Scala is now based on Scala 3. This is a completely different compiler ("dotty") and a quite different source language (we are using the classic Java-style syntax, not the new Python-style syntax). diff -r d7e0b6620c07 -r 06eb4d0031e3 etc/build.props --- a/etc/build.props Fri Aug 19 05:49:17 2022 +0000 +++ b/etc/build.props Sat Aug 20 21:34:55 2022 +0200 @@ -116,6 +116,7 @@ src/Pure/PIDE/command_span.scala \ src/Pure/PIDE/document.scala \ src/Pure/PIDE/document_id.scala \ + src/Pure/PIDE/document_info.scala \ src/Pure/PIDE/document_status.scala \ src/Pure/PIDE/editor.scala \ src/Pure/PIDE/headless.scala \ diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Algebra/README.html --- a/src/HOL/Algebra/README.html Fri Aug 19 05:49:17 2022 +0000 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,85 +0,0 @@ - - - - -
- -These proofs are mainly by Florian Kammüller. (Later, Larry -Paulson simplified some of the proofs.) These theories were indeed -the original motivation for locales. - -Here is an outline of the directory's contents:
Group
defines semigroups, monoids,
-groups, commutative monoids, commutative groups, homomorphisms and the
-subgroup relation. It also defines the product of two groups
-(This theory was reimplemented by Clemens Ballarin).
-
-FiniteProduct
extends
-commutative groups by a product operator for finite sets (provided by
-Clemens Ballarin).
-
-Coset
defines
-the factorization of a group and shows that the factorization a normal
-subgroup is a group.
-
-Bij
-defines bijections over sets and operations on them and shows that they
-are a group. It shows that automorphisms form a group.
-
-Exponent
the
- combinatorial argument underlying Sylow's first theorem.
-
-Sylow
-contains a proof of the first Sylow theorem.
-CRing
-defines Abelian monoids and groups. The difference to commutative
- structures is merely notational: the binary operation is
- addition rather than multiplication. Commutative rings are
- obtained by inheriting properties from Abelian groups and
- commutative monoids. Further structures in the algebraic
- hierarchy of rings: integral domain.
-
-Module
-introduces the notion of a R-left-module over an Abelian group, where
- R is a ring.
-
-UnivPoly
-constructs univariate polynomials over rings and integral domains.
- Degree function. Universal Property.
-A development of univariate polynomials for HOL's ring classes
-is available at HOL/Library/Polynomial
.
-
-
[Jacobson1985] Nathan Jacobson, Basic Algebra I, Freeman, 1985. - -
[Ballarin1999] Clemens Ballarin, Computer Algebra and Theorem Proving, - Author's PhD thesis, 1999. Also University of Cambridge, Computer Laboratory Technical Report number 473. - -
- - - diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Algebra/README.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Algebra/README.thy Sat Aug 20 21:34:55 2022 +0200 @@ -0,0 +1,74 @@ +theory README imports Main +begin + +section \The current development is built above the HOL (Higher-Order Logic) -Isabelle theory and the formalization of protocols introduced by Larry Paulson. More details are -in his paper -The Inductive approach -to verifying cryptographic protocols (J. Computer Security 6, pages -85-128, 1998). - -
-This directory contains a number of files: - -
Last modified 20 August 2002 - -
-Frederic Blanqui, -blanqui@lri.fr - - - diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Auth/Guard/README_Guard.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Auth/Guard/README_Guard.thy Sat Aug 20 21:34:55 2022 +0200 @@ -0,0 +1,57 @@ +theory README_Guard imports Main +begin + +section \Cryptographic protocols are of major importance, especially with the -growing use of the Internet. This directory demonstrates the ``inductive -method'' of protocol verification, which is described in various -papers. The operational semantics of protocol participants is defined -inductively. - -
This directory contains proofs concerning - -
Frederic Blanqui has contributed a theory of guardedness, which is -demonstrated by proofs of some roving agent protocols. - -
-Larry Paulson, -lcp@cl.cam.ac.uk - - - diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Auth/README.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Auth/README.thy Sat Aug 20 21:34:55 2022 +0200 @@ -0,0 +1,38 @@ +theory README imports Main +begin + +section \- -The most recent description of HOLCF is found here: - -
- -After loading theory Hoare, you can state goals of the form -
-VARS x y ... {P} prog {Q} --where prog is a program in the above language, P is the -precondition, Q the postcondition, and x y ... is the -list of all program variables in prog. The latter list must -be nonempty and it must include all variables that occur on the left-hand -side of an assignment in prog. Example: -
-VARS x {x = a} x := x+1 {x = a+1} --The (normal) variable a is merely used to record the initial -value of x and is not a program variable. Pre/post conditions -can be arbitrary HOL formulae mentioning both program variables and normal -variables. -
- -The implementation hides reasoning in Hoare logic completely and provides a -method vcg for transforming a goal in Hoare logic into an -equivalent list of verification conditions in HOL: -
-apply vcg --If you want to simplify the resulting verification conditions at the same -time: -
-apply vcg_simp --which, given the example goal above, solves it completely. For further -examples see Examples. -
- -IMPORTANT: -This is a logic of partial correctness. You can only prove that your program -does the right thing if it terminates, but not that it -terminates. -A logic of total correctness is also provided and described below. - -
- -A total-correctness goal has the form -
-VARS x y ... [P] prog [Q] --enclosing the pre- and postcondition in square brackets. -
- -Methods vcg_tc and vcg_tc_simp can be used to derive -verification conditions. -
- -From a total-correctness proof, a function can be extracted which -for every input satisfying the precondition returns an output -satisfying the postcondition. - -
-Mike Gordon.
-Mechanizing Programming Logics in Higher Order Logic.
-University of Cambridge, Computer Laboratory, TR 145, 1988.
-
-published as -
-Mike Gordon.
-Mechanizing Programming Logics in Higher Order Logic.
-In
-Current Trends in Hardware Verification and Automated Theorem Proving
-,
-edited by G. Birtwistle and P.A. Subrahmanyam, Springer-Verlag, 1989.
-
- -The main differences: the state is modelled as a tuple as suggested in -
-J. von Wright and J. Hekanaho and P. Luostarinen and T. Langbacka. -Mechanizing Some Advanced Refinement Concepts. -Formal Methods in System Design, 3, 1993, 49-81. -
-and the embeding is deep, i.e. there is a concrete datatype of programs. The
-latter is not really necessary.
-
-
diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Hoare/README.thy
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Hoare/README.thy Sat Aug 20 21:34:55 2022 +0200
@@ -0,0 +1,93 @@
+theory README imports Main
+begin
+
+section \
-
-Addition of new theories should be done with some care, as the
-``module system'' of Isabelle is rather simplistic. The following
-guidelines may be helpful to achieve maximum re-usability and minimum
-clashes with existing developments.
-
- This directory formalizes TLA in Isabelle/HOL, as follows:
-
-The theories are accompanied by a small number of examples:
-
-The directory presents verification examples involving program composition.
-They are mostly taken from the works of Chandy, Charpentier and Chandy.
-
- Safety proofs (invariants) are often proved automatically. Progress
-proofs involving ENSURES can sometimes be proved automatically. The
-level of automation appears to be about the same as in HOL-UNITY by Flemming
-Andersen et al.
-
-HOL-Library: supplemental theories for main Isabelle/HOL
-
-This is a collection of generic theories that may be used together
-with main Isabelle/HOL.
-
-
-
-
-
-
-
diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/Library/README.thy
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Library/README.thy Sat Aug 20 21:34:55 2022 +0200
@@ -0,0 +1,43 @@
+theory README imports Main
+begin
+
+section \TLA: Lamport's Temporal Logic of Actions
-
-TLA
-is a linear-time temporal logic introduced by Leslie Lamport in
-The Temporal Logic of Actions (ACM TOPLAS 16(3), 1994,
-872-923). Unlike other temporal logics, both systems and properties
-are represented as logical formulas, and logical connectives such as
-implication, conjunction, and existential quantification represent
-structural relations such as refinement, parallel composition, and
-hiding. TLA has been applied to numerous case studies.
-
-
-
-
-Please consult the
-design notes
-for further information regarding the setup and use of this encoding
-of TLA.
-
-
-
-
-
-
-
-Stephan Merz
-
-
-Last modified: Sat Mar 5 00:54:49 CET 2005
-
-
diff -r d7e0b6620c07 -r 06eb4d0031e3 src/HOL/TLA/README.thy
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/TLA/README.thy Sat Aug 20 21:34:55 2022 +0200
@@ -0,0 +1,48 @@
+theory README imports Main
+begin
+
+section \UNITY: Examples Involving Program Composition
-
-
-
-
-Counter.thy
)
-and priority system (Priority.thy
)
-
-Alloc.thy
)
-
-Client.thy
)
-
-AllocImpl.thy
)
-
-Handshake.thy
)
-
-TimerArray.thy
)
-