Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
merged
2009-11-20, by wenzelm
merged
2009-11-20, by nipkow
Rene tuned proof
2009-11-20, by nipkow
example theory for new domain package
2009-11-20, by huffman
thy_decl outer syntax for repdef
2009-11-19, by huffman
merged
2009-11-19, by huffman
nicer warning message for indirect-recursive domain definitions
2009-11-19, by huffman
store map_ID thms in theory data; automate proofs of reach lemmas
2009-11-19, by huffman
add map_ID lemmas
2009-11-19, by huffman
domain_isomorphism package defines combined copy function
2009-11-19, by huffman
merged
2009-11-20, by nipkow
added Rene Thiemann's normalize function
2009-11-20, by nipkow
added lemma
2009-11-20, by nipkow
merged
2009-11-19, by huffman
domain_isomorphism package defines copy functions
2009-11-19, by huffman
copy_of_dtyp uses map table from theory data
2009-11-19, by huffman
Domain.thy imports Representable.thy
2009-11-19, by huffman
fix definitions of copy combinators
2009-11-19, by huffman
clean up indentation; add 'definitional' option flag
2009-11-19, by huffman
rename generated abs_iso, rep_iso lemmas
2009-11-19, by huffman
clean up indentation
2009-11-19, by huffman
add dependency on domain_isomorphism.ML
2009-11-19, by huffman
set up domain_isomorphism package in Representable.thy
2009-11-19, by huffman
automate proofs of map_ID theorems
2009-11-19, by huffman
change Theory.requires
2009-11-19, by huffman
use theory data for REP_simps and isodefl_rules
2009-11-19, by huffman
replace defl_tab and map_tab with theory data
2009-11-19, by huffman
separate conjuncts of isodefl theorem
2009-11-19, by huffman
automate isodefl proof
2009-11-19, by huffman
change example to use recursion with continuous function space
2009-11-19, by huffman
add lemma isodefl_cprod
2009-11-19, by huffman
automate definition of map functions; remove unused code
2009-11-19, by huffman
change naming convention for deflation combinators
2009-11-19, by huffman
add new makefile dependencies
2009-11-19, by huffman
prove isomorphism and isodefl rules
2009-11-19, by huffman
avoid using csplit; define copy functions exactly like the current domain package
2009-11-19, by huffman
merged
2009-11-19, by huffman
remove one_typ and tr_typ; add abs/rep lemmas
2009-11-18, by huffman
automate definition of rep/abs functions
2009-11-18, by huffman
get rid of numbers on thy variables
2009-11-18, by huffman
automate proofs of REP equations
2009-11-18, by huffman
cleaned up; factored out fixed-point definition code
2009-11-18, by huffman
automate solution of domain equations
2009-11-18, by huffman
removed fixme - quick-and-dirty flag is appropriate
2009-11-20, by Christian Urban
use of thm-antiquotation
2009-11-20, by Christian Urban
Added new counterexample generator SML_inductive for goals involving
2009-11-19, by berghofe
Added infrastructure for embedding random data generators into code generated
2009-11-19, by berghofe
unused_thms: show only results from 'theorem(s)' package (via old-style kinds);
2009-11-19, by wenzelm
future_result: purge flexflex pairs, which should normally be trivial anyway -- prevent Thm.future_result from complaining about tpairs;
2009-11-19, by wenzelm
toplevel pretty printer for Synchronized.var;
2009-11-19, by wenzelm
adapted Local_Theory.define -- eliminated odd thm kind;
2009-11-19, by wenzelm
Specification.definition: Thm.definitionK marks exactly the high-level end-user result;
2009-11-19, by wenzelm
Local_Theory.define: eliminated slightly odd kind argument -- such low-level definitions should be hardly ever exposed to end-users anyway;
2009-11-19, by wenzelm
merged
2009-11-19, by wenzelm
merged
2009-11-19, by paulson
Minor correction
2009-11-19, by paulson
some attempts to improve termination of isatest;
2009-11-19, by wenzelm
Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
2009-11-19, by hoelzl
Renamed vector_less_eq_def to the more usual name vector_le_def.
2009-11-19, by hoelzl
merged
2009-11-19, by bulwahn
replacing Predicate_Compile_Preproc_Const_Defs by more general Spec_Rules
2009-11-19, by bulwahn
concealing internal definitions of primrec specifications
2009-11-19, by bulwahn
adding derived constant Predicate.holds to Predicate theory; adopting the predicate compiler
2009-11-19, by bulwahn
changing the proof procedure for parameters; adding a testcase for negation and parameters; adopting print_tac to the latest function print_tac' in the predicate compiler
2009-11-19, by bulwahn
adopting proposed_modes; adding a new dimension of complexity for nicer error messages; tuned
2009-11-19, by bulwahn
check if equations are present for all functions to avoid low-level exception later
2009-11-19, by krauss
anti_sym -> antisym
2009-11-19, by nipkow
optionally trace theorems used in proof reconstruction
2009-11-18, by boehmes
added arithmetic example using div and mod
2009-11-18, by boehmes
bump up Nitpick's axiom/definition unfolding limits, because some real-world problems (e.g. from Boogie) ran into the previous limits;
2009-11-17, by blanchet
merged
2009-11-17, by blanchet
comment out debugging code in Nitpick
2009-11-17, by blanchet
fixed bug in Nitpick's handling of "The" and "Eps" when the return type is a "bool"
2009-11-17, by blanchet
made "NitpickHOL.normalized_rhs_of" more robust in the face of locale definitions
2009-11-17, by blanchet
removed "debug := true" that shouldn't have been submitted in the first place
2009-11-17, by blanchet
Added derivation and Brouwer's fixpoint theorem in Multivariate Analysis (translated by Robert Himmelmann from HOL-light)
2009-11-17, by hoelzl
merged
2009-11-17, by blanchet
run Nitpick examples if Kodkodi is available
2009-11-17, by blanchet
merged
2009-11-17, by wenzelm
fixed "expect" of Nitpick examples to reflect latest changes in Nitpick
2009-11-17, by blanchet
merged
2009-11-17, by blanchet
use SAT solver that's available everywhere for this example
2009-11-17, by blanchet
invoke Kodkodi from Nitpick using new $KODKOD/bin/kodkodi script;
2009-11-17, by blanchet
merged
2009-11-17, by blanchet
added constraint for Eq^- in Nitpick's implementation of the monotonicity calculus
2009-11-16, by blanchet
change the order in which Nitpick tries SAT solvers;
2009-11-16, by blanchet
Fixed splitting of div and mod on integers (split theorem differed from implementation).
2009-11-17, by webertj
merged
2009-11-17, by webertj
Fixed splitting of div and mod on integers (split theorem differed from implementation).
2009-11-17, by webertj
init_theory: Runtime.controlled_execution for proper exception trace etc.;
2009-11-17, by wenzelm
eliminated slightly odd name space grouping -- now managed by Isar toplevel;
2009-11-17, by wenzelm
implicit name space grouping for theory/local_theory transactions;
2009-11-17, by wenzelm
uniform new_group/reset_group;
2009-11-17, by wenzelm
eliminated dead code;
2009-11-17, by wenzelm
generalized procs for rewrite_proof: allow skeleton;
2009-11-16, by wenzelm
member/cons: slightly more correct treatment of multi-index, notably empty one;
2009-11-16, by wenzelm
merged
2009-11-16, by wenzelm
Fixed a typo in a comment.
2009-11-16, by webertj
Fixed a typo in a comment.
2009-11-16, by webertj
merged
2009-11-16, by paulson
A few more lemmas from Jeremy
2009-11-16, by paulson
removed hassize predicate
2009-11-16, by hoelzl
Added new lemmas to Euclidean Space by Robert Himmelmann
2009-11-16, by hoelzl
eliminated obsolete thm position stuff;
2009-11-16, by wenzelm
tuned signature;
2009-11-16, by wenzelm
guard future proofs by Goal.future_enabled;
2009-11-16, by wenzelm
further explosion of HOL-Boogie verification conditions
2009-11-16, by boehmes
merged
2009-11-16, by haftmann
proper purge
2009-11-16, by haftmann
dropped obsolete documentation; updated generated sources
2009-11-16, by haftmann
merged
2009-11-16, by blanchet
removed a few global names in Nitpick (styp, nat_less, pairf)
2009-11-13, by blanchet
add_expand_thm: explicit indication of is_def instead of fragile heuristic, tuned signature;
2009-11-15, by wenzelm
axiomatization: declare Spec_Rules, direct result;
2009-11-15, by wenzelm
use simultaneous Morphics.fact;
2009-11-15, by wenzelm
primitive defs: clarified def (axiom name) vs. description;
2009-11-15, by wenzelm
eliminated obsolete thm position tags;
2009-11-15, by wenzelm
permissive AList.merge -- most likely setup for theory data (beware of spurious AList.DUP);
2009-11-15, by wenzelm
provide actual Nitpick_HOL.extended_context;
2009-11-15, by wenzelm
tuned;
2009-11-15, by wenzelm
more accurate dependencies;
2009-11-15, by wenzelm
eliminated obsolete CVS Ids;
2009-11-15, by wenzelm
merged
2009-11-15, by schirmer
added benchmark for large records
2009-11-15, by schirmer
merged
2009-11-14, by schirmer
clarified quick-and-dirty usage in record package;
2009-11-14, by schirmer
simplified bulky metis proofs;
2009-11-15, by wenzelm
properly inlined @{lemma} antiqutations -- might also reduce proof terms a bit;
2009-11-15, by wenzelm
moved old SList, LList, LFilter to AFP/Lazy-Lists-II;
2009-11-14, by wenzelm
include HOL-Boogie keywords by default;
2009-11-14, by wenzelm
eliminated obsolete CVS Ids;
2009-11-14, by wenzelm
updated keywords;
2009-11-14, by wenzelm
generate keywords for Emacs Proof General only;
2009-11-14, by wenzelm
dismantled remains of old jEdit plugin;
2009-11-14, by wenzelm
isabelle_document: more explicit error output, notably for drafts;
2009-11-14, by wenzelm
LocalTheory -> Local_Theory
2009-11-13, by huffman
merged
2009-11-13, by huffman
automate definition of representable domains from algebraic deflations
2009-11-13, by huffman
cleaned up, removed unneeded call to Syntax.check_term
2009-11-13, by huffman
merged
2009-11-13, by nipkow
moved lemma from Algebra/IntRing to Ring_and_Field
2009-11-13, by nipkow
merged
2009-11-13, by wenzelm
merged
2009-11-13, by nipkow
-
2009-11-13, by nipkow
updated Local_Theory and Theory_Target;
2009-11-13, by wenzelm
modernized structure Local_Theory;
2009-11-13, by wenzelm
eliminated slightly odd kind argument of LocalTheory.note(s);
2009-11-13, by wenzelm
inductive: eliminated obsolete kind;
2009-11-13, by wenzelm
merged
2009-11-13, by paulson
A little rationalisation
2009-11-13, by paulson
eliminated obsolete "generated" kind -- collapsed to unspecific "" (definitely unused according to Lukas Bulwahn);
2009-11-13, by wenzelm
merged
2009-11-13, by boehmes
removed unused code and unused arguments,
2009-11-13, by boehmes
adapted proofs due to changes in HOL-Boogie
2009-11-13, by boehmes
parallel solving of Boogie splinters
2009-11-13, by boehmes
corrected translation of integer operators,
2009-11-13, by boehmes
extended theory simpset to simplify non-linear problems
2009-11-13, by boehmes
more "anti_sym" -> "antisym" (cf. a4179bf442d1);
2009-11-13, by wenzelm
merged
2009-11-13, by nipkow
renamed lemmas "anti_sym" -> "antisym"
2009-11-13, by nipkow
a few lemmas for point-free reasoning about transitive closure
2009-11-13, by krauss
merged
2009-11-13, by paulson
A number of theorems contributed by Jeremy Avigad
2009-11-13, by paulson
merged
2009-11-13, by bulwahn
merged
2009-11-12, by bulwahn
adding the predicate compiler quickcheck to the ex/ROOT.ML; adopting this quickcheck to the latest changes
2009-11-12, by bulwahn
removed annoying tracing message
2009-11-12, by bulwahn
added a tabled implementation of the reflexive transitive closure
2009-11-12, by bulwahn
merged
2009-11-12, by huffman
merged
2009-11-12, by huffman
improved ML interface to pcpodef
2009-11-12, by huffman
use Drule.standard (following typedef package), add pcpodef tactic interface
2009-11-11, by huffman
eliminated slightly odd (unused) "axiom" and "assumption" -- collapsed to unspecific "";
2009-11-12, by wenzelm
eliminated obsolete "internal" kind -- collapsed to unspecific "";
2009-11-12, by wenzelm
unused_thms: ignore kind -- already observes "concealed" flag;
2009-11-12, by wenzelm
all_valid_thms: more sophisticated check against global + local name space;
2009-11-12, by wenzelm
Remove map_compose, replaced by map_map
2009-11-12, by hoelzl
New list theorems; added map_map to simpset, this is the prefered direction; allow sorting by a key
2009-11-12, by hoelzl
Renamed upd_snd_conv to apsnd_conv to be consistent with apfst_conv; Added apsnd_apfst_commute
2009-11-12, by hoelzl
merged
2009-11-12, by haftmann
accomplish mutual recursion between fun and inst
2009-11-12, by haftmann
moved lemma map_of_zip_map to Map.thy
2009-11-12, by haftmann
merged
2009-11-12, by haftmann
explicit code lemmas produce nices code
2009-11-12, by haftmann
repaired broken code_const for term_of [String.literal]
2009-11-12, by haftmann
fixed soundness bug in Nitpick related to sets
2009-11-12, by blanchet
removed unnecessary oracle in the predicate compiler
2009-11-12, by bulwahn
improving code quality thanks to Florian's code review
2009-11-12, by bulwahn
renaming code_pred_intros to code_pred_intro
2009-11-12, by bulwahn
announcing the predicate compiler in NEWS and CONTRIBUTORS
2009-11-12, by bulwahn
new names for predicate functions in the predicate compiler
2009-11-12, by bulwahn
removed deprecated mode annotation parser; renamed accepted mode annotation parser to nicer naming
2009-11-12, by bulwahn
added another example to the predicate compiler
2009-11-12, by bulwahn
changed modes to expected_modes; added UNION to code_pred_inlining; fixed some examples; tuned
2009-11-12, by bulwahn
removed dummy setup for predicate compiler commands as the compiler is now part of HOL-Main
2009-11-12, by bulwahn
adopted predicate compiler examples to new syntax for modes
2009-11-12, by bulwahn
added interface of user proposals for names of generated constants
2009-11-12, by bulwahn
first steps towards a new mode datastructure; new syntax for mode annotations and new output of modes
2009-11-12, by bulwahn
adding more tests for the values command; adding some forbidden constants to inductify
2009-11-12, by bulwahn
Enables tests for locale functionality that is now available.
2009-11-11, by ballarin
merged
2009-11-11, by wenzelm
uniform use of simultabeous use_thys;
2009-11-11, by wenzelm
merged
2009-11-11, by haftmann
explicit invocation of code generation
2009-11-11, by haftmann
adding code equations for constructors
2009-11-11, by haftmann
tuned
2009-11-11, by haftmann
changed URL of SMT server,
2009-11-11, by boehmes
Added two new lemmas
2009-11-11, by paulson
tuned imports
2009-11-11, by haftmann
tuned
2009-11-11, by haftmann
local mutex for theory content/identity operations;
2009-11-11, by wenzelm
admit dummy implementation;
2009-11-11, by wenzelm
Toplevel.thread provides Isar-style exception output;
2009-11-10, by wenzelm
generalized Runtime.toplevel_error wrt. output function;
2009-11-10, by wenzelm
exported SimpleThread.attributes;
2009-11-10, by wenzelm
plain add_preference, no setmp_CRITICAL required;
2009-11-10, by wenzelm
adapted Theory_Data;
2009-11-10, by wenzelm
recovered update from 7264824baf66, which got lost in 7264824baf66;
2009-11-10, by wenzelm
merged
2009-11-10, by wenzelm
merged
2009-11-10, by haftmann
tuned header
2009-11-10, by haftmann
substantial simplification restores code generation
2009-11-10, by haftmann
lemmas about apfst and apsnd
2009-11-10, by haftmann
tuned imports
2009-11-10, by haftmann
merged
2009-11-10, by huffman
HOLCF example: domain package proofs done manually
2009-11-10, by huffman
add lemma parallel_fix_ind
2009-11-10, by huffman
add title/author block
2009-11-10, by huffman
theory of representable cpos
2009-11-10, by huffman
add map_map lemmas
2009-11-09, by huffman
add in_deflation relation, more lemmas about cast
2009-11-09, by huffman
ep_pair and deflation lemmas for powerdomain map functions
2009-11-09, by huffman
remove spurious parameter to "merge"
2009-11-10, by blanchet
merged, and renamed local "TheoryData" to "Data" (following common Isabelle conventions)
2009-11-10, by blanchet
fixed soundness bug in Nitpick related to sets of sets;
2009-11-10, by blanchet
added possibility to register datatypes as codatatypes in Nitpick;
2009-11-05, by blanchet
added datatype constructor cache in Nitpick (to speed up the scope enumeration) and never test more than 4096 scopes
2009-11-05, by blanchet
don't promise too much in the Nitpick manual
2009-11-05, by blanchet
merged
2009-11-05, by blanchet
added "nitpick_def" attribute to lfp/gfp definition generated by the inductive package;
2009-11-05, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip