Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+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.
tuned;
2007-08-30, by wenzelm
moved type_mode to type.ML;
2007-08-30, by wenzelm
infer_types: general check_typs instead of Type.cert_typ_mode;
2007-08-30, by wenzelm
maintain mode in context (get/set/restore_mode);
2007-08-30, by wenzelm
added burrow_types;
2007-08-30, by wenzelm
- tuned section about inductive predicates
2007-08-30, by berghofe
ported div/mod simprocs from HOL/ex/Binary.thy
2007-08-30, by huffman
renamed POLYML_LINK_OPTIONS to POLY_LINK_OPTIONS;
2007-08-29, by wenzelm
added POLYML_LINK_OPTIONS, which is required for unusual platforms (notably cygwin);
2007-08-29, by wenzelm
some simultaneous use_thys;
2007-08-29, by wenzelm
Updated section about inductive definitions.
2007-08-29, by berghofe
turned list comprehension translations into ML to optimize base case
2007-08-29, by nipkow
added Hoare/hoare_tac.ML (code from Hoare/Hoare.thy, also required in Isar_examples/Hoare.thy);
2007-08-29, by wenzelm
added x86-solaris;
2007-08-29, by wenzelm
fixed Proofs
2007-08-29, by chaieb
added Hoare/hoare_tac.ML (code from Hoare/Hoare.thy, also required in Isar_examples/Hoare.thy);
2007-08-29, by wenzelm
removed unused theorems ; added lifting properties for foldr and foldl
2007-08-29, by chaieb
removed Hoare/hoare.ML, Hoare/hoareAbort.ML, ex/svc_oracle.ML (which can be mistaken as attached ML script on case-insensitive file-system);
2007-08-29, by wenzelm
Deleted unused fillin_mixfix function.
2007-08-29, by berghofe
mark all parallel sessions as experimental
2007-08-29, by kleing
atbroy99 is 64bit
2007-08-29, by kleing
fixed pattern comnpletion; untabified
2007-08-28, by krauss
revert to Word library version from 2007/08/20
2007-08-28, by huffman
TheoremHook: fixed copy-paste mistake;
2007-08-28, by wenzelm
Smaller size and fewer iterations for quickcheck.
2007-08-28, by berghofe
codegen.ML is now loaded in Pure again.
2007-08-28, by berghofe
Changed "code" attribute of concat_map_singleton to "code unfold".
2007-08-28, by berghofe
Code generator now uses sequences with depth limit.
2007-08-28, by berghofe
Got rid of large simpset in proof of characteristic equations
2007-08-28, by berghofe
Added sequences with recursion depth limit.
2007-08-28, by berghofe
Adapted to changes in interface of Specification.theorem_i
2007-08-28, by berghofe
- restored old setup
2007-08-28, by berghofe
codegen.ML is now loaded in Pure again.
2007-08-28, by berghofe
- new auto-quickcheck flag
2007-08-28, by berghofe
Added local_theory_to_proof'
2007-08-28, by berghofe
- theorem(_i) now also takes "interactive" flag as argument
2007-08-28, by berghofe
Specification.theorem now also takes "interactive" flag as argument.
2007-08-28, by berghofe
Commented out non-standard paragraph formatting.
2007-08-28, by nipkow
added (code) lemmas for setsum and foldl
2007-08-28, by nipkow
replaced 'sorry' by unproven;
2007-08-28, by wenzelm
do not touch quick_and_dirty;
2007-08-28, by wenzelm
norm_absolute: CRITICAL;
2007-08-28, by wenzelm
tuned load order -- minimizes modules before Secure;
2007-08-28, by wenzelm
induct: proper separation of initial and terminal step;
2007-08-28, by wenzelm
move WordExamples to Examples directory
2007-08-28, by huffman
HOL-Word-Examples
2007-08-28, by huffman
Word Examples directory
2007-08-28, by huffman
add parallel sessions for atbroy99 and macbroy6
2007-08-28, by kleing
HOL_USEDIR_OPTIONS: no special -M setting (now works with multithreaded);
2007-08-27, by wenzelm
Added infinite_descent
2007-08-27, by nipkow
updated keywords
2007-08-27, by haftmann
added code_props
2007-08-27, by haftmann
introduces params_of_sort
2007-08-27, by haftmann
added simple definition scheme
2007-08-27, by haftmann
added explicit equation for equality of nested environments
2007-08-27, by haftmann
circumvented infix problem
2007-08-27, by haftmann
tuned linear arith (once again) with ring_distribs
2007-08-26, by nipkow
made SML/NJ happy
2007-08-26, by haftmann
described 'rotated' attribute
2007-08-26, by kleing
made SML/NJ happy
2007-08-25, by haftmann
revised blacklisting for ATP linkup
2007-08-24, by paulson
new derived rule: incr_type_indexes
2007-08-24, by paulson
Returning both a "one-line" proof and a structured proof
2007-08-24, by paulson
Reconstruction bug fix
2007-08-24, by paulson
overloaded definitions accompanied by explicit constants
2007-08-24, by haftmann
moved class dense_linear_order to Orderings.thy
2007-08-24, by haftmann
updated
2007-08-24, by haftmann
made sets executable
2007-08-24, by haftmann
remove unused lemmas
2007-08-24, by huffman
bin_sc_nth proof
2007-08-24, by huffman
remove lemma bin_rec_PM
2007-08-23, by huffman
avoid use of bin_rec_PM
2007-08-23, by huffman
new instance proofs
2007-08-23, by huffman
remove unused lemmas
2007-08-23, by huffman
import BinInduct;
2007-08-23, by huffman
declare bin_rest_BIT_bin_last [simp]
2007-08-23, by huffman
Word/BinInduct.thy
2007-08-23, by huffman
theory of integers as an inductive datatype
2007-08-23, by huffman
move bin_nth stuff to its own subsection
2007-08-23, by huffman
removed Word/Size.thy;
2007-08-22, by huffman
typed print translation for CARD('a);
2007-08-22, by huffman
rename type pls to num0
2007-08-22, by huffman
move constant definitions to their respective subsections
2007-08-22, by huffman
tuned;
2007-08-22, by chaieb
More selective generalization : a*b is generalized whenever none of a and b is a number
2007-08-22, by chaieb
imports Presburger; no need for Main
2007-08-22, by chaieb
move bool list operations from WordBitwise to WordBoolList
2007-08-22, by huffman
Word/WordBoolList.thy
2007-08-22, by huffman
move if_simps from BinBoolList to Num_Lemmas
2007-08-22, by huffman
Axioms for class no longer use object-universal quantifiers
2007-08-22, by chaieb
move bool list stuff from WordDefinition and WordArith to new WordBoolList theory
2007-08-22, by huffman
move bool list stuff from BinOperations to BinBoolList;
2007-08-22, by huffman
Added mod cancellation simproc
2007-08-21, by nipkow
remove redundant lemmas
2007-08-21, by huffman
declare conj_absorb [simp]
2007-08-21, by huffman
replace iszero_number_of_Pls with iszero_0 in rel_simps
2007-08-21, by huffman
add lemma of_int_power
2007-08-21, by huffman
Isar-style proof for lfp_ordinal_induct
2007-08-21, by huffman
ProofContext.restore_mode;
2007-08-21, by wenzelm
added inner syntax mode, includes former type_mode and is_stmt;
2007-08-21, by wenzelm
Modified message for sendback
2007-08-21, by paulson
"sendback" to PG for one-line proof reconstructions
2007-08-21, by paulson
Deleted the partially-typed translation and the combinator code.
2007-08-21, by paulson
move BIT datatype stuff from Num_Lemmas to BinGeneral
2007-08-21, by huffman
simplify termination proof
2007-08-21, by huffman
simplify proof of word_of_int
2007-08-21, by huffman
improved evaluation interface
2007-08-21, by haftmann
moved ordered_ab_semigroup_add to OrderedGroup.thy
2007-08-21, by haftmann
updated
2007-08-21, by haftmann
move udvd, div and mod stuff from WordDefinition to WordArith
2007-08-21, by huffman
move order-related stuff from WordDefinition to WordArith
2007-08-21, by huffman
add lemma one_less_power
2007-08-21, by huffman
move scast/ucast stuff to its own subsection
2007-08-21, by huffman
move shifting-related constant definitions from WordDefinition to WordShift
2007-08-21, by huffman
use HOL-ex later;
2007-08-21, by wenzelm
standard_parse_term: added pp/check argument, include disambig here (from sign.ML);
2007-08-20, by wenzelm
inner syntax: added parse_term/prop;
2007-08-20, by wenzelm
read_def_terms: moved disambig to syntax.ML;
2007-08-20, by wenzelm
tuned CRITICAL sections;
2007-08-20, by wenzelm
remove redundant lemma int_number_of
2007-08-20, by huffman
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip