History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Statespace/distinct_tree_prover.ML
Revision Date Author Comments
# 81b459a5 08-Apr-2016 wenzelm <none@none>

eliminated unused simproc identifier;


# b97bf4c0 23-Feb-2016 nipkow <none@none>

more canonical names


# e0a30cbb 09-Sep-2015 wenzelm <none@none>

simplified simproc programming interfaces;


# 7f7de75b 18-Jul-2015 wenzelm <none@none>

prefer tactics with explicit context;


# 9a9cf694 05-Jul-2015 wenzelm <none@none>

simplified Thm.instantiate and derivatives: the LHS refers to non-certified variables -- this merely serves as index into already certified structures (or is ignored);


# 6d5ce04c 03-Jul-2015 wenzelm <none@none>

clarified context;


# b8ef3466 01-Jun-2015 wenzelm <none@none>

clarified context;


# 740a17d4 06-Mar-2015 wenzelm <none@none>

Thm.cterm_of and Thm.ctyp_of operate on local context;


# 5f318eee 04-Mar-2015 wenzelm <none@none>

clarified signature;


# 34035ccd 04-Mar-2015 wenzelm <none@none>

tuned signature -- prefer qualified names;


# 1a2798f1 07-Mar-2014 wenzelm <none@none>

removed dead code;


# 0928b2db 18-Apr-2013 wenzelm <none@none>

simplifier uses proper Proof.context instead of historic type simpset;


# 79a4e2f9 12-Apr-2013 wenzelm <none@none>

tuned exceptions -- avoid composing error messages in low-level situations;


# 941cf8eb 02-Dec-2011 wenzelm <none@none>

more antiquotations;


# 201045de 06-Nov-2011 wenzelm <none@none>

inlined antiquotations;


# 197b731c 06-Nov-2011 wenzelm <none@none>

misc tuning and modernization;


# 9c72c6e0 29-Jun-2011 wenzelm <none@none>

simplified/unified Simplifier.mk_solver;


# 7cfe82ef 16-Apr-2011 wenzelm <none@none>

proper subgoal addressing via SUBGOAL/CSUBGOAL -- assuming these tactics did not handle Subscript in any special way;
tuned;


# 6d2612c8 16-Apr-2011 wenzelm <none@none>

modernized structure Proof_Context;


# 27ff3609 06-Sep-2010 wenzelm <none@none>

more antiquotations;


# b11705e1 28-Aug-2010 haftmann <none@none>

formerly unnamed infix equality now named HOL.eq


# 2ab2e08e 25-Aug-2010 wenzelm <none@none>

renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;


# 33076e76 19-Aug-2010 haftmann <none@none>

tuned quotes


# bbda5041 19-Aug-2010 haftmann <none@none>

use antiquotations for remaining unqualified constants in HOL


# 628125bc 15-May-2010 wenzelm <none@none>

tuned;


# e3d0611a 27-Feb-2010 wenzelm <none@none>

modernized structure Term_Ord;


# da1c433c 05-Mar-2009 wenzelm <none@none>

removed spurious occurrences of old rep_ss;


# 20840102 01-Jan-2009 wenzelm <none@none>

normalized some ML type/val aliases;


# e154e805 31-Dec-2008 wenzelm <none@none>

moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
tuned signature of structure Term;


# b91805aa 10-Dec-2008 wenzelm <none@none>

more antiquotations;


# a6513468 19-Mar-2008 wenzelm <none@none>

simplified get_thm(s): back to plain name argument;


# a46b31e4 19-Mar-2008 wenzelm <none@none>

renamed datatype thmref to Facts.ref, tuned interfaces;


# 1fc22904 12-Nov-2007 schirmer <none@none>

added signatures;
tuned


# d93a6fb8 24-Oct-2007 schirmer <none@none>

added Statespace library