History log of /seL4-l4v-master/l4v/lib/MonadicRewrite.thy
Revision Date Author Comments
# a45adef6 31-Oct-2020 Gerwin Klein <gerwin.klein@data61.csiro.au>

all: remove theory import path references

In Isabelle2020, when isabelle jedit is started without a session
context, e.g. `isabelle jedit -l ASpec`, theory imports with path
references cause the isabelle process to hang.

Since sessions now declare directories, Isabelle can find those files
without path reference and we therefore remove all such path references
from import statements. With this, `jedit` and `build` should work with
and without explicit session context as before.

Signed-off-by: Gerwin Klein <gerwin.klein@data61.csiro.au>


# a424d55e 09-Mar-2020 Gerwin Klein <gerwin.klein@data61.csiro.au>

licenses: convert license tags to SPDX


# 21cc25f1 19-Nov-2018 Edward Pierzchalski <ed.pierzchalski@data61.csiro.au>

lib: Add stray lemmas and methods.

These were unused items in ARM CRefine, now kept for potential future
usefulness.


# 1ae3a8d6 20-Jun-2018 Gerwin Klein <gerwin.klein@data61.csiro.au>

Isabelle2018: Lib update


# 6b9d9d24 09-Jun-2018 Gerwin Klein <gerwin.klein@data61.csiro.au>

Isabelle2018: new "op x" syntax; now is "(x)"

(result of "isabelle update_op -m <dir>")


# d4996217 13-Jun-2018 Rafal Kolanski <rafal.kolanski@nicta.com.au>

lib: add generic lemmas from SELFOUR-584 updates

Mainly concerning word_ctz and enumeration_both.


# 877312f0 24-Nov-2017 Rafal Kolanski <rafal.kolanski@nicta.com.au>

lib: generic/word/monad/hoare lemmas from SELFOUR-242 verification

Notably useful is hoare_vcg_lift_imp' which generates an implication
rather than a disjunction.

Monadic rewrite rules should be modified to preserve bound variable
names, as demonstrated by monadic_rewrite_symb_exec_l'_preserve_names.
Addressing this more comprehensively is left as a TODO item for the
future (see VER-554).


# 796887d9 11-Jul-2017 Alejandro Gomez-Londono <alejandro.gomez@nicta.com.au>

Removes all trailing whitespaces


# 47119bf4 13-Jan-2017 Gerwin Klein <gerwin.klein@nicta.com.au>

wp_cleanup: update proofs for new wp behaviour

The things that usually go wrong:
- wp fall through: add +, e.g.
apply (wp select_wp) -> apply (wp select_wp)+

- precondition: you can remove most hoare_pre, but wpc still needs it, and
sometimes the wp instance relies on being able to fit a rule to the
current non-schematic precondition. In that case, use "including no_pre"
to switch off the automatic hoare_pre application.

- very rarely there is a schematic postcondition that interferes with the
new trivial cleanup rules, because the rest of the script assumes some
specific state afterwards (shouldn't happen in a reasonable proof, but
not all proofs are reasonable..). In that case, (wp_once ...)+ should
emulate the old behaviour precisely.


# 41d4aa4f 25-Oct-2016 Matthew Brecknell <Matthew.Brecknell@data61.csiro.au>

Isabelle2016-1: update references to renamed constants and facts


# 879ac302 09-Nov-2016 Alejandro Gomez-Londono <alejandro.gomez@nicta.com.au>

Lib: Addition of auxiliary lemmas in basic theories to better support CRefine

* Generalized version of bind_inv_inv_comm for easier swapping inside
the nondet monad

* New ccorres_symb_exec_r_known_rv

* New zip_take lemmas for handling `take n (zip x y)` situations

tags: [VER-623][SELFOUR-413]


# f0faa90f 17-Apr-2016 Gerwin Klein <gerwin.klein@nicta.com.au>

lib/spec/proof/tools: fix word change fallout


# 671c5673 27-Jan-2016 Miki Tanaka <miki.tanaka@nicta.com.au>

more fixes in DRefine: some changes in proofs involving uint / unat


# 65e1f39a 30-Nov-2015 Japheth Lim <Japheth.Lim@nicta.com.au>

autocorres-crefine: update CRefine with new corres_UL.


# 375b526b 01-Dec-2015 Thomas Sewell <Thomas.Sewell@nicta.com.au>

Finally done with array assertions.


# e8d1ed6d 09-Aug-2014 Gerwin Klein <gerwin.klein@nicta.com.au>

ported lib/* theories to Isabelle2014-RC0


# 1af1d2b6 08-Aug-2014 Gerwin Klein <gerwin.klein@nicta.com.au>

some of the global Isabelle2014 renames

option_case -> case_option
sum_case -> case_sum
prod_case -> case_prod
Option.set -> set_option
Option.map -> map_option
option_rel -> rel_option
list_all2_def -> list_all2_iff
map.simps -> list.map
tl.simps -> list.sel(2-3)
the.simps -> option.sel


# 84595f42 17-Jul-2014 Gerwin Klein <gerwin.klein@nicta.com.au>

release cleanup


# 2a03e81d 14-Jul-2014 Gerwin Klein <gerwin.klein@nicta.com.au>

Import release snapshot.