Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
transform_error: pass through Interrupt;
2002-08-08, by wenzelm
tuned;
2002-08-08, by wenzelm
exception SIMPROC_FAIL: solid error reporting of simprocs;
2002-08-08, by wenzelm
tuned prove_conv (error reporting done within meta_simplifier.ML);
2002-08-08, by wenzelm
adhoc_freeze_vars;
2002-08-08, by wenzelm
proper instantiation of mk_left_commute;
2002-08-08, by wenzelm
converted;
2002-08-08, by wenzelm
tuned deps;
2002-08-08, by wenzelm
use Tactic.prove instead of prove_goalw_cterm in internal proofs!
2002-08-08, by wenzelm
Tactic.prove, Tactic.prove_standard;
2002-08-08, by wenzelm
* Pure: improved error reporting of simprocs;
2002-08-08, by wenzelm
tuned;
2002-08-07, by wenzelm
mk_left_commute: proper instantiation avoids expensive unification;
2002-08-07, by wenzelm
tuned;
2002-08-07, by wenzelm
Simplifier.simproc(_i);
2002-08-07, by wenzelm
Added time example at the end.
2002-08-07, by nipkow
section on "Rule declarations and methods";
2002-08-07, by wenzelm
Removed (now unneeded) declaration of realizer for induction on datatype b.
2002-08-07, by berghofe
Removed (now unneeded) declarations of realizers for induction on lists and letters.
2002-08-07, by berghofe
Added file Tools/datatype_realizer.ML
2002-08-07, by berghofe
Removed (now unneeded) declaration of realizers for induction on natural numbers.
2002-08-07, by berghofe
Module for defining realizers for induction and case analysis theorems
2002-08-07, by berghofe
Added calls to add_dt_realizers.
2002-08-07, by berghofe
Exported function make_tnames.
2002-08-07, by berghofe
Fixed two bugs
2002-08-07, by nipkow
* Provers: Simplifier.simproc(_i) now provide sane interface for
2002-08-06, by wenzelm
sane interface for simprocs;
2002-08-06, by wenzelm
fixed intern_skolem: disallow internal names (why didn't anybody notice?!?);
2002-08-06, by wenzelm
predefined locales "var" and "struct" (useful for sharing parameters);
2002-08-06, by wenzelm
* Pure: predefined locales "var" and "struct" are useful for sharing
2002-08-06, by wenzelm
protect simplifier operation against spurious exceptions from simprocs;
2002-08-05, by wenzelm
tuned;
2002-08-05, by wenzelm
special syntax for index "1" (plain numeral hidden by "1" symbol in HOL);
2002-08-05, by wenzelm
Removed theory NatDef.
2002-08-05, by berghofe
Replaced nat_ind_tac by induct_tac.
2002-08-05, by berghofe
Removed proof of Suc_le_D (already proved in Nat.thy).
2002-08-05, by berghofe
Removed reference to theory NatDef.
2002-08-05, by berghofe
Removed reference to simpset of NatDef.thy
2002-08-05, by berghofe
Legacy ML bindings.
2002-08-05, by berghofe
- Converted to new theory format
2002-08-05, by berghofe
Moved NatDef stuff to theory Nat.
2002-08-05, by berghofe
updated;
2002-08-05, by wenzelm
added Isabelle LNCSes;
2002-08-02, by wenzelm
fixed long statement: P.opt_thm_name;
2002-08-02, by wenzelm
fixed railroads;
2002-08-02, by wenzelm
typedef: "open" option;
2002-08-02, by wenzelm
declare projected "axioms" as "elim?";
2002-08-02, by wenzelm
better satisfies rules for is_recfun
2002-08-01, by paulson
some progress towards "satisfies"
2002-07-31, by paulson
*** empty log message ***
2002-07-31, by nipkow
added mk_left_commute to HOL.thy and used it "everywhere"
2002-07-31, by nipkow
separate "axioms" proofs: more flexible for locale reasoning
2002-07-31, by paulson
tweaks involving Separation
2002-07-31, by paulson
new theorem eq_commute
2002-07-31, by paulson
better sats rules for higher-order operators
2002-07-30, by paulson
removal of twos_compl.ML, which is not really needed
2002-07-30, by paulson
- changed date format for proper lexicographical ordering
2002-07-30, by isatest
changed date format for proper lexicographical ordering
2002-07-30, by isatest
tuned messages;
2002-07-29, by wenzelm
tuned;
2002-07-29, by wenzelm
eliminate open locales and special ML code;
2002-07-29, by wenzelm
tuned document;
2002-07-28, by wenzelm
make SML/NJ happy;
2002-07-27, by wenzelm
support for split assumptions in cases (hyps vs. prems);
2002-07-26, by wenzelm
tuned;
2002-07-26, by wenzelm
More lemmas, working towards relativization of "satisfies"
2002-07-25, by paulson
Added the assumption nth_replacement to locale M_datatypes.
2002-07-25, by paulson
simplified locale predicates;
2002-07-24, by wenzelm
removed unused locale_facts(_i);
2002-07-24, by wenzelm
tuned;
2002-07-24, by wenzelm
tweaks, aiming towards relativization of "satisfies"
2002-07-24, by paulson
Tuned type constraint of function merge_rules to make smlnj happy.
2002-07-24, by berghofe
AC18: meta-level predicate via locale;
2002-07-24, by wenzelm
tuned view;
2002-07-24, by wenzelm
removed attribute "norm_hhf";
2002-07-24, by wenzelm
adapted fact names;
2002-07-24, by wenzelm
predicate defs via locales;
2002-07-24, by wenzelm
locales: predicate defs;
2002-07-24, by wenzelm
* Pure: locale specifications now produce predicate definitions;
2002-07-24, by wenzelm
Relativization and Separation for the function "nth"
2002-07-23, by paulson
Added "nocite" to avoid BibTeX error when proofs are switched off.
2002-07-22, by berghofe
Added program extraction keywords.
2002-07-21, by berghofe
Document for program extraction in HOL.
2002-07-21, by berghofe
Examples for program extraction in HOL.
2002-07-21, by berghofe
Rules for rewriting HOL proofs.
2002-07-21, by berghofe
Added theory for setting up program extraction.
2002-07-21, by berghofe
Added program extraction module.
2002-07-21, by berghofe
*** empty log message ***
2002-07-19, by wenzelm
accomodate cumulative locale predicates;
2002-07-19, by wenzelm
support locale ``views'' (for cumulative predicates);
2002-07-19, by wenzelm
Towards relativization and absoluteness of formula_rec
2002-07-19, by paulson
Absoluteness of the function "nth"
2002-07-19, by paulson
A couple of new theorems for Constructible
2002-07-19, by paulson
absoluteness for "formula" and "eclose"
2002-07-18, by paulson
define cumulative predicate view;
2002-07-18, by wenzelm
adapted add_locale;
2002-07-18, by wenzelm
adapted locale syntax;
2002-07-18, by wenzelm
fixed inform_file_retracted: remove_thy;
2002-07-18, by wenzelm
ACe_axioms;
2002-07-18, by wenzelm
added satisfy_hyps;
2002-07-18, by wenzelm
quantify LC (conflict with const name of HOL);
2002-07-18, by wenzelm
new theorems to support Constructible proofs
2002-07-18, by paulson
Formulas (and lists) in M (and L!)
2002-07-17, by paulson
Expressing Lset and L without using length and arity; simplifies Separation
2002-07-17, by paulson
Added conditional and (&&) and or (||).
2002-07-16, by schirmer
adapted locales;
2002-07-16, by wenzelm
adapted locales;
2002-07-16, by wenzelm
tuned;
2002-07-16, by wenzelm
adapted locales;
2002-07-16, by wenzelm
rearranged to work without proof contexts;
2002-07-16, by wenzelm
export_standard supercedes export_single;
2002-07-16, by wenzelm
export map_context;
2002-07-16, by wenzelm
assert_propT;
2002-07-16, by wenzelm
proper predicate definitions of locale body;
2002-07-16, by wenzelm
add_locale: adapted args;
2002-07-16, by wenzelm
locale: optional predicate name, or "open";
2002-07-16, by wenzelm
module now right after ProofContext (for locales);
2002-07-16, by wenzelm
avoid "_st" versions of proof data;
2002-07-16, by wenzelm
context rules;
2002-07-16, by wenzelm
tuned order of modules;
2002-07-16, by wenzelm
added equal_elim_rule1;
2002-07-16, by wenzelm
moved stuff to List.thy;
2002-07-16, by wenzelm
moved stuff from Main.thy;
2002-07-16, by wenzelm
adapted to locale defs;
2002-07-16, by wenzelm
updated;
2002-07-16, by wenzelm
instantiation of locales M_trancl and M_wfrank;
2002-07-16, by paulson
tweaked definition of setclass
2002-07-16, by paulson
new lemmas
2002-07-16, by paulson
*** empty log message ***
2002-07-16, by nipkow
mail address update
2002-07-15, by isatest
fix latex output
2002-07-15, by schirmer
Removal of mono.thy
2002-07-14, by paulson
improved presentation markup
2002-07-14, by paulson
merged Update with func
2002-07-14, by paulson
little Bugfix
2002-07-12, by schirmer
towards relativization of "iterates" and "wfrec"
2002-07-12, by paulson
new definitions of fun_apply and M_is_recfun
2002-07-12, by paulson
*** empty log message ***
2002-07-11, by nipkow
tidied
2002-07-11, by paulson
Added "using" to the beginning of original newman proof again, because
2002-07-11, by berghofe
Separation/Replacement up to M_wfrank!
2002-07-11, by paulson
*** empty log message ***
2002-07-11, by nipkow
Added partly automated version of Newman.
2002-07-11, by nipkow
Fixed markup error in comment.
2002-07-11, by schirmer
*** empty log message ***
2002-07-11, by nipkow
*** empty log message ***
2002-07-11, by nipkow
expand_proof now also takes an optional term describing the proposition
2002-07-10, by berghofe
- Moved abs_def to drule.ML
2002-07-10, by berghofe
Simplified proof of induction rule for datatypes involving function types.
2002-07-10, by berghofe
Fixed quantified variable name preservation for ball and bex (bounded quants)
2002-07-10, by paulson
*** empty log message ***
2002-07-10, by nipkow
Added unary and binary operations like (+,-,<, ...); Added smallstep semantics (no proofs about it yet).
2002-07-10, by schirmer
tuned add_thmss;
2002-07-10, by wenzelm
tuned Locale.add_thmss;
2002-07-10, by wenzelm
added assert_judgment;
2002-07-10, by wenzelm
NameSpace.accesses';
2002-07-10, by wenzelm
added accesses';
2002-07-10, by wenzelm
tuned;
2002-07-10, by wenzelm
*** empty log message ***
2002-07-10, by nipkow
*** empty log message ***
2002-07-10, by nipkow
better document preparation
2002-07-09, by paulson
converted List to new-style
2002-07-09, by paulson
*** empty log message ***
2002-07-09, by nipkow
Added function abs_def.
2002-07-09, by berghofe
more and simpler separation proofs
2002-07-09, by paulson
More relativization, reflection and proofs of separation
2002-07-09, by paulson
*** empty log message ***
2002-07-09, by nipkow
tuned;
2002-07-09, by wenzelm
send email plaform independently
2002-07-09, by isatest
More Separation proofs
2002-07-09, by paulson
new files
2002-07-09, by paulson
*** empty log message ***
2002-07-08, by nipkow
more and simpler separation proofs
2002-07-08, by paulson
tuned;
2002-07-08, by wenzelm
Defining a meta-existential quantifier.
2002-07-08, by paulson
*** empty log message ***
2002-07-08, by nipkow
*** empty log message ***
2002-07-08, by nipkow
*** empty log message ***
2002-07-08, by nipkow
*** empty log message ***
2002-07-08, by nipkow
reflection for more internal formulas
2002-07-08, by paulson
clarified text content of locale body;
2002-07-08, by wenzelm
*** empty log message ***
2002-07-08, by nipkow
more internalized formulas and separation proofs
2002-07-05, by paulson
*** empty log message ***
2002-07-05, by nipkow
more separation instances
2002-07-05, by paulson
for ZF document
2002-07-05, by paulson
fixed precedences of **
2002-07-05, by paulson
added dependency for $(OUT)/Pure
2002-07-05, by kleing
added dependency for $(OUT)/FOL
2002-07-05, by kleing
More use of relativized quantifiers
2002-07-04, by paulson
Constructible: some separation axioms
2002-07-04, by paulson
tuned;
2002-07-04, by wenzelm
Constructible/document/root.tex;
2002-07-04, by wenzelm
document setup;
2002-07-04, by wenzelm
*** empty log message ***
2002-07-04, by nipkow
tweaks
2002-07-04, by paulson
reflection for rall and rex
2002-07-04, by paulson
towards proving separation for L
2002-07-04, by paulson
separation of M_axioms into M_triv_axioms and M_axioms
2002-07-04, by paulson
miniscoping for class-bounded quantifiers (rall and rex)
2002-07-04, by paulson
fixed comment;
2002-07-03, by wenzelm
added a list search example.
2002-07-03, by nipkow
conversion of QUniv to Isar
2002-07-02, by paulson
conversion of QPair to Isar
2002-07-02, by paulson
thms_containing: optional limit argument;
2002-07-02, by wenzelm
proper treatment of border cases;
2002-07-02, by wenzelm
tuned print_thms_containing;
2002-07-02, by wenzelm
update thms_containing;
2002-07-02, by wenzelm
* improved thms_containing: proper indexing of facts instead of raw
2002-07-02, by wenzelm
removed thms_containing (see pure_thy.ML and proof_context.ML);
2002-07-02, by wenzelm
print_thms_containing: index variables, refer to local facts as well;
2002-07-02, by wenzelm
these_facts: refrain from put_thmss (2nd time!);
2002-07-02, by wenzelm
ProofContext.pretty_fact;
2002-07-02, by wenzelm
tuned msg;
2002-07-02, by wenzelm
improved thms_containing (use FactIndex.T etc.);
2002-07-02, by wenzelm
ProofContext.print_thms_containing;
2002-07-02, by wenzelm
emulate old thms_containing;
2002-07-02, by wenzelm
added fact_index.ML;
2002-07-02, by wenzelm
Facts indexed by consts or (some) frees.
2002-07-02, by wenzelm
Tidying and introduction of various new theorems
2002-07-02, by paulson
more use of relativized quantifiers
2002-07-01, by paulson
*** empty log message ***
2002-07-01, by nipkow
modified Larry's changes to make div/mod a numeral work in arith.
2002-07-01, by nipkow
*** empty log message ***
2002-07-01, by nipkow
less
more
|
(0)
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip