History log of /seL4-l4v-10.1.1/isabelle/src/ZF/UNITY/Constrains.thy
Revision Date Author Comments
# 274ed9c2 20-May-2018 wenzelm <none@none>

avoid undeclared frees;


# 8ecffcf0 23-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


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

prefer tactics with explicit context;


# b8d56fe6 10-Feb-2015 wenzelm <none@none>

proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
occasionally clarified use of context;


# 4eae0352 10-Nov-2014 wenzelm <none@none>

proper context for assume_tac (atac remains as fall-back without context);


# 2257dcda 02-Nov-2014 wenzelm <none@none>

modernized header;


# db5aeb3c 16-Aug-2014 wenzelm <none@none>

prefer 'named_theorems' over Named_Thms, with subtle change of semantics due to visual order vs. internal reverse order;


# 63a76875 14-Dec-2013 wenzelm <none@none>

proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
clarified tool context in some boundary cases;


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

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


# f5cf0e45 06-Mar-2012 paulson <none@none>

More mathematical symbols for ZF examples


# 29168e90 20-Nov-2011 wenzelm <none@none>

eliminated obsolete "standard";


# 50fe8111 28-Oct-2011 wenzelm <none@none>

tuned Named_Thms: proper binding;


# 2f53d74a 13-May-2011 wenzelm <none@none>

proper Proof.context for classical tactics;
reduced claset to snapshot of classical context;
discontinued clasimpset;


# 2b1723df 28-Feb-2010 wenzelm <none@none>

more antiquotations;
eliminated legacy ML bindings;


# 079cde2d 17-Oct-2009 wenzelm <none@none>

eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;


# a4b600c4 23-Jul-2009 wenzelm <none@none>

renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;


# 7b41de27 02-Jul-2009 wenzelm <none@none>

renamed NamedThmsFun to Named_Thms;
simplified/unified names of instances of Named_Thms;


# b1258973 16-Mar-2009 wenzelm <none@none>

simplified method setup;


# 77d6b267 13-Mar-2009 wenzelm <none@none>

unified type Proof.method and pervasive METHOD combinators;


# e7a16ceb 07-Oct-2007 wenzelm <none@none>

modernized specifications;
removed legacy ML bindings;


# a1538a69 29-Jul-2007 wenzelm <none@none>

replaced program_defs_ref by proper context data (via attribute "program");


# 95ee7518 21-Jul-2007 wenzelm <none@none>

tactics: avoid dynamic reference to accidental theory context (via ML_Context.the_context etc.);


# ba766b3f 03-Jul-2007 wenzelm <none@none>

rewrite_goal_tac;


# 9989d06d 06-Dec-2006 wenzelm <none@none>

reorganized structure Goal vs. Tactic;


# f7800759 29-Nov-2006 wenzelm <none@none>

simplified method setup;


# b0eed312 02-Jun-2005 paulson <none@none>

renamed "constrains" to "safety" to avoid keyword clash


# 13a8140b 28-Mar-2005 paulson <none@none>

conversion of UNITY to Isar scripts


# dd2a5068 27-May-2003 paulson <none@none>

updating ZF-UNITY with Sidi's new material


# 3184becc 15-Nov-2001 ehmety <none@none>

*** empty log message ***


# 59a188ae 08-Aug-2001 paulson <none@none>

new ZF/UNITY theory