krauss [Wed, 23 Sep 2009 13:48:35 +0200] rev 32654
atbroy101 is long dead, use atbroy99; comment out broken SML test invocation
haftmann [Wed, 23 Sep 2009 13:42:53 +0200] rev 32653
merged
haftmann [Wed, 23 Sep 2009 12:03:47 +0200] rev 32652
stripped legacy ML bindings
hoelzl [Wed, 23 Sep 2009 13:31:38 +0200] rev 32651
Undo errornous commit of Statespace change
hoelzl [Wed, 23 Sep 2009 13:17:17 +0200] rev 32650
correct variable order in approximate-method
paulson [Wed, 23 Sep 2009 11:06:32 +0100] rev 32649
merged
paulson [Wed, 23 Sep 2009 11:05:28 +0100] rev 32648
Correct chasing of type variable instantiations during type unification.
The following theory should not raise exception TERM:
constdefs
somepredicate :: "(('b => 'b) => ('a => 'a))
=> 'a => 'b => bool"
"somepredicate upd v x == True"
lemma somepredicate_idI:
"somepredicate id (f v) v"
by (simp add: somepredicate_def)
lemma somepredicate_triv:
"somepredicate upd v x ==> somepredicate upd v x"
by assumption
lemmas somepredicate_triv [OF somepredicate_idI]
lemmas st' = somepredicate_triv[where v="h :: nat => bool"]
lemmas st2 = st'[OF somepredicate_idI]
haftmann [Wed, 23 Sep 2009 11:33:52 +0200] rev 32647
hide newly introduced constants
Philipp Meyer [Tue, 22 Sep 2009 11:26:46 +0200] rev 32646
used standard fold function and type aliases
Philipp Meyer [Mon, 21 Sep 2009 15:05:26 +0200] rev 32645
sos method generates and uses proof certificates